aboutsummaryrefslogtreecommitdiff
path: root/src/BoundedArithmetic/Double/Proofs/ShiftLeftRightTactic.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/BoundedArithmetic/Double/Proofs/ShiftLeftRightTactic.v')
-rw-r--r--src/BoundedArithmetic/Double/Proofs/ShiftLeftRightTactic.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/src/BoundedArithmetic/Double/Proofs/ShiftLeftRightTactic.v b/src/BoundedArithmetic/Double/Proofs/ShiftLeftRightTactic.v
index 44b4eb36d..997fb1937 100644
--- a/src/BoundedArithmetic/Double/Proofs/ShiftLeftRightTactic.v
+++ b/src/BoundedArithmetic/Double/Proofs/ShiftLeftRightTactic.v
@@ -1,7 +1,8 @@
Require Import Coq.ZArith.ZArith.
Require Import Crypto.BoundedArithmetic.Interface.
Require Import Crypto.Util.ZUtil.
-Require Import Crypto.Util.Tactics.
+Require Import Crypto.Util.Tactics.UniquePose.
+Require Import Crypto.Util.Tactics.BreakMatch.
Local Open Scope Z_scope.