aboutsummaryrefslogtreecommitdiff
path: root/src/LegacyArithmetic/Pow2Base.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/LegacyArithmetic/Pow2Base.v')
-rw-r--r--src/LegacyArithmetic/Pow2Base.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/src/LegacyArithmetic/Pow2Base.v b/src/LegacyArithmetic/Pow2Base.v
index 62f1f742d..c5c69e684 100644
--- a/src/LegacyArithmetic/Pow2Base.v
+++ b/src/LegacyArithmetic/Pow2Base.v
@@ -1,6 +1,5 @@
Require Import Coq.ZArith.Zpower Coq.ZArith.ZArith.
Require Import Crypto.Util.ListUtil.
-Require Import Crypto.Util.ZUtil.
Require Import Coq.Lists.List.
Local Open Scope Z_scope.