From 5384ed9ab7557c515c8522b0229f10663e5a3161 Mon Sep 17 00:00:00 2001 From: herbelin Date: Fri, 10 Feb 2006 08:44:40 +0000 Subject: code mort git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8022 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Init/Logic.v | 10 ---------- 1 file changed, 10 deletions(-) (limited to 'theories/Init/Logic.v') diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v index 7d9884505..cefbb989d 100755 --- a/theories/Init/Logic.v +++ b/theories/Init/Logic.v @@ -230,16 +230,6 @@ Section Logic_lemmas. End equality. -(* Is now a primitive principle - Theorem eq_rect: (A:Type)(x:A)(P:A->Type)(P x)->(y:A)(eq ? x y)->(P y). - Proof. - Intros. - Cut (identity A x y). - NewDestruct 1; Auto. - NewDestruct H; Auto. - Qed. -*) - Definition eq_ind_r : forall (A:Type) (x:A) (P:A -> Prop), P x -> forall y:A, y = x -> P y. intros A x P H y H0; elim sym_eq with (1 := H0); assumption. -- cgit v1.2.3