aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/Eqdep.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-04 15:58:49 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-04 15:58:49 +0000
commitbb02036b476d3a3e7b3b79568257ef3d28ea6a11 (patch)
treec328cc8913aa1db6f3c7c1f85a1f26185986c15c /theories/Logic/Eqdep.v
parentdb9beee355f93cc6403d1837dc9674d20ebce30e (diff)
Mise en conformité nouveau Simpl pour Fix
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@654 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/Eqdep.v')
-rwxr-xr-xtheories/Logic/Eqdep.v8
1 files changed, 5 insertions, 3 deletions
diff --git a/theories/Logic/Eqdep.v b/theories/Logic/Eqdep.v
index d1f45be08..86fd7c9ec 100755
--- a/theories/Logic/Eqdep.v
+++ b/theories/Logic/Eqdep.v
@@ -46,7 +46,7 @@ Lemma eq_dep_dep1 : (p,q:U)(x:(P p))(y:(P q))(eq_dep p x q y)->(eq_dep1 p x q y)
Proof.
Induction 1; Intros.
Apply eq_dep1_intro with (refl_equal U p).
-Elim eq_rec_eq; Trivial.
+Simpl. Trivial.
Qed.
Lemma eq_dep1_eq : (p:U)(x,y:(P p))(eq_dep1 p x p y)->x=y.
@@ -60,7 +60,7 @@ Proof.
Intros; Apply eq_dep1_eq; Apply eq_dep_dep1; Trivial.
Qed.
-Lemma equiv_eqex_eqdep : (p,q:U)(x:(P p))(y:(P q))
+Lemma equiv_eqex_eq_dep : (p,q:U)(x:(P p))(y:(P q))
(existS U P p x)=(existS U P q y) <-> (eq_dep p x q y).
Proof.
Split.
@@ -79,13 +79,15 @@ Elim H.
Auto.
Qed.
+(* For compatibility *)
+Syntactic Definition equiv_eqex_eqdep := equiv_eqex_eq_dep.
Lemma inj_pair2: (p:U)(x,y:(P p))
(existS U P p x)=(existS U P p y)-> x=y.
Proof.
Intros.
Apply eq_dep_eq.
-Generalize (equiv_eqex_eqdep p p x y) .
+Generalize (equiv_eqex_eq_dep p p x y) .
Induction 1.
Intros.
Auto.