aboutsummaryrefslogtreecommitdiff
path: root/src/Reflection/Z/Reify.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Reflection/Z/Reify.v')
-rw-r--r--src/Reflection/Z/Reify.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Reflection/Z/Reify.v b/src/Reflection/Z/Reify.v
index 3c42c162c..451e522d0 100644
--- a/src/Reflection/Z/Reify.v
+++ b/src/Reflection/Z/Reify.v
@@ -9,7 +9,7 @@ Require Import Crypto.Reflection.InlineInterp.
Require Import Crypto.Reflection.Linearize.
Require Import Crypto.Reflection.LinearizeInterp.
-Ltac base_reify_op op op_head ::=
+Ltac base_reify_op op op_head extra ::=
lazymatch op_head with
| @Z.add => constr:(reify_op op op_head 2 Add)
| @Z.mul => constr:(reify_op op op_head 2 Mul)