aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/EqdepFacts.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-03-30 06:56:50 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-03-30 06:56:50 +0000
commit3b681990a903e3e71c3bea663685482ec170d558 (patch)
tree4d2896ee9ef1b8f9997a19d7ae6d734f5237438a /theories/Logic/EqdepFacts.v
parente7c20952e90d4f70ae84ab60b6aab62691c18aa0 (diff)
Réajout de eq_rec_eq oublié lors de la modularisation de Eqdep
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8674 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/EqdepFacts.v')
-rw-r--r--theories/Logic/EqdepFacts.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/theories/Logic/EqdepFacts.v b/theories/Logic/EqdepFacts.v
index 32237a0c9..167ba7839 100644
--- a/theories/Logic/EqdepFacts.v
+++ b/theories/Logic/EqdepFacts.v
@@ -302,6 +302,10 @@ Lemma eq_rect_eq :
forall (p:U) (Q:U -> Type) (x:Q p) (h:p = p), x = eq_rect p Q x p h.
Proof M.eq_rect_eq U.
+Lemma eq_rec_eq :
+ forall (p:U) (Q:U -> Set) (x:Q p) (h:p = p), x = eq_rect p Q x p h.
+Proof (fun p Q => M.eq_rect_eq U p Q).
+
(** Injectivity of Dependent Equality *)
Lemma eq_dep_eq : forall (P:U->Type) (p:U) (x y:P p), eq_dep p x p y -> x = y.