From 969cb56234750c320768ae39e934b18ce2883aef Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Fri, 10 Jun 2016 16:43:21 -0400 Subject: 8.5 fixes --- src/Testbit.v | 3 ++- 1 file changed, 2 insertions(+), 1 deletion(-) (limited to 'src/Testbit.v') 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. -- cgit v1.2.3