aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Tactics/DebugPrint.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Util/Tactics/DebugPrint.v')
-rw-r--r--src/Util/Tactics/DebugPrint.v4
1 files changed, 3 insertions, 1 deletions
diff --git a/src/Util/Tactics/DebugPrint.v b/src/Util/Tactics/DebugPrint.v
index 3ced23331..97edd0ad9 100644
--- a/src/Util/Tactics/DebugPrint.v
+++ b/src/Util/Tactics/DebugPrint.v
@@ -1,3 +1,5 @@
+Require Import Crypto.Util.Tactics.ConstrFail.
+
Ltac debuglevel := constr:(0%nat).
Ltac solve_debugfail tac :=
@@ -36,7 +38,7 @@ Ltac constr_run_tac_fail tac :=
let dummy := match goal with
| _ => tac ()
end in
- constr:(I : I).
+ constr_fail.
Ltac cidtac msg :=
constr_run_tac ltac:(fun _ => idtac msg).