aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Equality.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Util/Equality.v')
-rw-r--r--src/Util/Equality.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/src/Util/Equality.v b/src/Util/Equality.v
index 04335dbd4..d1a711821 100644
--- a/src/Util/Equality.v
+++ b/src/Util/Equality.v
@@ -8,6 +8,13 @@ Require Import Coq.Classes.Morphisms.
Require Import Crypto.Util.Isomorphism.
Require Import Crypto.Util.HProp.
+Import EqNotations.
+
+Definition f_equal_dep {A B} (f : forall a : A, B a) (x y : A) (H : x = y) : rew [B] H in f x = f y
+ := match H with
+ | eq_refl => eq_refl
+ end.
+
(** Most of the structure of proofs of equalities fits into what
mathematicians call a weak ∞-groupoid. (In fact, one way of
*defining* a weak ∞-groupoid is via what's called the J-rule,