aboutsummaryrefslogtreecommitdiff
path: root/src/Testbit.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-06-10 16:43:21 -0400
committerGravatar Jason Gross <jgross@mit.edu>2016-06-10 16:43:21 -0400
commit969cb56234750c320768ae39e934b18ce2883aef (patch)
tree50ceed23e66d66f635d671929f5330f52159defa /src/Testbit.v
parentecf5f6fc0d3107eeb8566f56037f28d888a53a1a (diff)
8.5 fixes
Diffstat (limited to 'src/Testbit.v')
-rw-r--r--src/Testbit.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/src/Testbit.v b/src/Testbit.v
index 264069587..2bfcc3df6 100644
--- a/src/Testbit.v
+++ b/src/Testbit.v
@@ -3,6 +3,7 @@ Require Import Crypto.Util.ListUtil Crypto.Util.CaseUtil Crypto.Util.ZUtil.
Require Import Crypto.BaseSystem Crypto.BaseSystemProofs.
Require Import Coq.ZArith.ZArith Coq.ZArith.Zdiv.
Require Import Coq.omega.Omega Coq.Numbers.Natural.Peano.NPeano Coq.Arith.Arith.
+Import Nat.
Local Open Scope Z.
@@ -209,4 +210,4 @@ Lemma testbit_spec : forall n us base limb_width, (0 < limb_width)%nat ->
Proof.
intros.
erewrite unfold_bits_testbit, unfold_bits_decode; eauto; omega.
-Qed. \ No newline at end of file
+Qed.