aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-02-21 20:42:52 -0500
committerGravatar Jason Gross <jgross@mit.edu>2017-05-28 09:38:36 -0400
commit1f705c9010a7a84d04ff393ac43d5af8e308dd81 (patch)
tree97cda7fd983571e600b31bd563760f898d5f3a82 /theories/Init
parent954a125f4470cf7d723cd78b003a4cf8c17ca3f6 (diff)
Use [rew_] instead of [eq_rect_] prefix
As per Hugo's request.
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 12ec9dd77..d6076f86d 100644
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -527,13 +527,13 @@ destruct e, e'.
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),
+Lemma eq_trans_rew_distr : forall A (P:A -> Type) (x y z:A) (e:x=y) (e':y=z) (k:P x),
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),
+Lemma rew_const : forall A P (x y:A) (e:x=y) (k:P),
rew [fun _ => P] e in k = k.
Proof.
destruct e; reflexivity.