aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Init')
-rw-r--r--theories/Init/Logic.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index 437d802d8..12ec9dd77 100644
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -528,13 +528,13 @@ reflexivity.
Defined.
Lemma eq_trans_eq_rect_distr : forall A (P:A -> Type) (x y z:A) (e:x=y) (e':y=z) (k:P x),
- eq_rect _ P k _ (eq_trans e e') = eq_rect _ P (eq_rect _ P k _ e) _ e'.
+ rew (eq_trans e e') in k = rew e' in rew e in k.
Proof.
destruct e, e'; reflexivity.
Defined.
Lemma eq_rect_const : forall A P (x y:A) (e:x=y) (k:P),
- eq_rect _ (fun _ : A => P) k _ e = k.
+ rew [fun _ => P] e in k = k.
Proof.
destruct e; reflexivity.
Defined.