aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic
diff options
context:
space:
mode:
authorGravatar Abhishek Anand <abhishek.anand.iitg@gmail.com>2016-12-11 11:59:33 -0500
committerGravatar GitHub <noreply@github.com>2016-12-11 11:59:33 -0500
commitd7abadbef61ab0d45ffc5a5a45ff31bd39103446 (patch)
tree37f13e8e56641a432b105a92578ed526d8d4d614 /theories/Logic
parentad768e435a736ca51ac79a575967b388b34918c7 (diff)
strengthened the statement of JMeq_eq_dep
because P:U->Prop implies P:U->Type, the new statement is strictly more useful. No change was needed to the proof.
Diffstat (limited to 'theories/Logic')
-rw-r--r--theories/Logic/JMeq.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Logic/JMeq.v b/theories/Logic/JMeq.v
index 2f95856b4..86d05e8fb 100644
--- a/theories/Logic/JMeq.v
+++ b/theories/Logic/JMeq.v
@@ -130,7 +130,7 @@ Qed.
is as strong as [eq_dep U P p x q y] (this uses [JMeq_eq]) *)
Lemma JMeq_eq_dep :
- forall U (P:U->Prop) p q (x:P p) (y:P q),
+ forall U (P:U->Type) p q (x:P p) (y:P q),
p = q -> JMeq x y -> eq_dep U P p x q y.
Proof.
intros.