aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-05-14 14:10:23 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-05-14 14:10:23 +0000
commit590512e3f003f0bdc26d585e996dc065936c7d4a (patch)
treee69d7e858a123b42e97e3fb38fdd90ffbb9ff189 /theories/Init
parent2799dbf2fe45d83f2a2828442735db0f0fb3d1d5 (diff)
ajout des theoremes eqT_rec_r et eqT_rect_r pour Rewrite
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2680 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init')
-rwxr-xr-xtheories/Init/Logic_Type.v10
1 files changed, 6 insertions, 4 deletions
diff --git a/theories/Init/Logic_Type.v b/theories/Init/Logic_Type.v
index af5b04ed0..fa375ad10 100755
--- a/theories/Init/Logic_Type.v
+++ b/theories/Init/Logic_Type.v
@@ -94,17 +94,19 @@ End Equality_is_a_congruence.
Hints Immediate sym_eqT sym_not_eqT : core v62.
-(** This states the replacement of equals by equals in a proposition *)
+(** This states the replacement of equals by equals *)
-Definition eqT_ind_r : (A:Type)(x:A)(P:A->Prop)(P x)->(y:A)(eqT ? y x)->(P y).
+Definition eqT_ind_r : (A:Type)(x:A)(P:A->Prop)(P x)->(y:A)y==x -> (P y).
Intros A x P H y H0; Case sym_eqT with 1:=H0; Trivial.
Defined.
-(** not allowed because of dependencies: [[
Definition eqT_rec_r : (A:Type)(x:A)(P:A->Set)(P x)->(y:A)y==x -> (P y).
Intros A x P H y H0; Case sym_eqT with 1:=H0; Trivial.
Defined.
-]] *)
+
+Definition eqT_rect_r : (A:Type)(x:A)(P:A->Type)(P x)->(y:A)y==x -> (P y).
+Intros A x P H y H0; Case sym_eqT with 1:=H0; Trivial.
+Defined.
(** Some datatypes at the [Type] level *)