aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/Eqdep.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-06 12:28:10 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-06 12:28:10 +0000
commitb40af3a0f07153f96fedef6092362b26fe191dfa (patch)
treea61255917817a3dacb8105cf04f96113894f69ac /theories/Logic/Eqdep.v
parent1e4655347b5704cc98709f69c1c0fd05e2cc9e15 (diff)
Un usage en moins de l'axiome eq_rec_eq
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@665 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/Eqdep.v')
-rwxr-xr-xtheories/Logic/Eqdep.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Logic/Eqdep.v b/theories/Logic/Eqdep.v
index d1f45be08..6f19c543b 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.