coq-club AT inria.fr
Subject: The Coq mailing list
List archive
Re: [Coq-Club]Problems proving equality of proof terms of inductively defined predicate.
chronological Thread
- From: David Nowak <david.nowak AT aist.go.jp>
- To: eelis AT eelis.net
- Cc: coq-club AT pauillac.inria.fr
- Subject: Re: [Coq-Club]Problems proving equality of proof terms of inductively defined predicate.
- Date: Fri, 09 Jun 2006 11:13:45 +0900
- List-archive: <http://pauillac.inria.fr/pipermail/coq-club/>
Hi Eelis,
You can prove Abis below which is a bit more general than A and then apply it. eq_rect is used to convince Coq that, because 0=n, C0 in also of type P n.
Require Export Eqdep_dec.
Inductive P : nat -> Prop := C0 : P 0 | C1 : P 1.
Lemma Abis : forall n (x : P n) (p : 0 = n), x = eq_rect 0 P C0 n p.
Proof.
intros n x.
case x.
intro.
pattern p in |- *.
apply K_dec_set.
decide equality.
reflexivity.
intro.
absurd (0 = 1).
discriminate.
assumption.
Qed.
Theorem A: forall (x: P 0), x = C0.
Proof.
intro.
apply (Abis 0 x (refl_equal 0)).
Qed.
Eelis van der Weegen a écrit :
Greetings.
Is the following provable? If it is, how? If it isn't, why not? :
Inductive P : nat -> Prop := C0 : P 0 | C1 : P 1.
Theorem A: forall (x: P 0), x = C0.
David
--
David Nowak
http://staff.aist.go.jp/david.nowak/
- [Coq-Club]Problems proving equality of proof terms of inductively defined predicate., Eelis van der Weegen
- Re: [Coq-Club]Problems proving equality of proof terms of inductively defined predicate., Roland Zumkeller
- Re: [Coq-Club]Problems proving equality of proof terms of inductively defined predicate., David Nowak
Archive powered by MhonArc 2.6.16.