aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Curry.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Util/Curry.v')
-rw-r--r--src/Util/Curry.v10
1 files changed, 2 insertions, 8 deletions
diff --git a/src/Util/Curry.v b/src/Util/Curry.v
index 8a34cb611..d1e3a7b94 100644
--- a/src/Util/Curry.v
+++ b/src/Util/Curry.v
@@ -1,14 +1,8 @@
+Require Import Crypto.Util.Tactics.ChangeInAll.
+
Definition curry2 {A B C} (f : A -> B -> C) (x : A * B) : C
:= let '(a, b) := x in f a b.
-(** Work around "Cannot create self-referring hypothesis" coming from
- [change x with y in *] *)
-Local Ltac change_in_all from to :=
- change from with to;
- repeat match goal with
- | [ H : _ |- _ ] => progress change from with to in H
- end.
-
Ltac change_with_curried f :=
cbv beta in f; (* work around https://coq.inria.fr/bugs/show_bug.cgi?id=5430 *)
lazymatch type of f with