aboutsummaryrefslogtreecommitdiff
path: root/src/LegacyArithmetic/Double/Proofs/ShiftLeftRightTactic.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/LegacyArithmetic/Double/Proofs/ShiftLeftRightTactic.v')
-rw-r--r--src/LegacyArithmetic/Double/Proofs/ShiftLeftRightTactic.v11
1 files changed, 10 insertions, 1 deletions
diff --git a/src/LegacyArithmetic/Double/Proofs/ShiftLeftRightTactic.v b/src/LegacyArithmetic/Double/Proofs/ShiftLeftRightTactic.v
index 41234bf6e..98cf3cf9c 100644
--- a/src/LegacyArithmetic/Double/Proofs/ShiftLeftRightTactic.v
+++ b/src/LegacyArithmetic/Double/Proofs/ShiftLeftRightTactic.v
@@ -1,8 +1,17 @@
Require Import Coq.ZArith.ZArith.
Require Import Crypto.LegacyArithmetic.Interface.
-Require Import Crypto.Util.ZUtil.
+Require Import Crypto.Util.ZUtil.Notations.
+Require Import Crypto.Util.ZUtil.Definitions.
+Require Import Crypto.Util.ZUtil.Testbit.
+Require Import Crypto.Util.ZUtil.Tactics.RewriteModSmall.
+Require Import Crypto.Util.ZUtil.Tactics.LtbToLt.
+Require Import Crypto.Util.ZUtil.Tactics.Ztestbit.
Require Import Crypto.Util.Tactics.UniquePose.
Require Import Crypto.Util.Tactics.BreakMatch.
+Require Export Crypto.Util.ZUtil.ZSimplify.Autogenerated.
+Require Export Crypto.Util.ZUtil.ZSimplify.Core.
+Require Export Crypto.Util.ZUtil.ZSimplify.Simple.
+Require Export Crypto.Util.ZUtil.LandLorShiftBounds.
Local Open Scope Z_scope.