coq-club AT inria.fr
Subject: The Coq mailing list
List archive
- From: casteran AT labri.fr
- To: coq-club AT pauillac.inria.fr
- Subject: [Coq-Club] (no subject)
- Date: Fri, 17 Sep 2004 18:17:57 +0200
- List-archive: <http://pauillac.inria.fr/pipermail/coq-club/>
Hello all,
Below is a simple proof that the only vector of length 0 is
Vnil. But this proof uses the axiom JMeq_eq. Is there any axiom-free
proof of the same result ?
Pierre
Require Import Bvector.
Require Import JMeq.
Lemma pim: forall (n:nat)(v:vector bool n), n=0 -> JMeq v (Vnil bool).
intros n v; case v.
reflexivity.
discriminate 1.
Qed.
Lemma pam: forall (v:vector bool 0), JMeq v (Vnil bool).
intro v; apply pim.
trivial.
Qed.
Lemma poum : forall (v:vector bool 0), eq v (Vnil bool).
intros v.
apply JMeq_eq.
apply pam.
Qed.
----------------------------------------------------------------
This message was sent using IMP, the Internet Messaging Program.
- [Coq-Club] (no subject), casteran
- Re: [Coq-Club] (no subject), Nicolas Magaud
- Re: [Coq-Club] (no subject), Thery Laurent
Archive powered by MhonArc 2.6.16.