aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ZUtil.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-05-12 13:11:37 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-05-12 13:11:37 -0400
commit59ea974cfae7041fd312195ee5c2b39c94e29e1b (patch)
tree7676849bf91a9975fb55a1e9e2a8aa8d6a2a9f64 /src/Util/ZUtil.v
parent05b86acbe41f8f98ebc2ce93ae3401cb6ff08a60 (diff)
Split off notation and defs in ZUtil
Diffstat (limited to 'src/Util/ZUtil.v')
-rw-r--r--src/Util/ZUtil.v10
1 files changed, 3 insertions, 7 deletions
diff --git a/src/Util/ZUtil.v b/src/Util/ZUtil.v
index bb19e6170..8e3d34ce4 100644
--- a/src/Util/ZUtil.v
+++ b/src/Util/ZUtil.v
@@ -11,13 +11,11 @@ Require Import Crypto.Util.Bool.
Require Import Crypto.Util.Notations.
Require Import Coq.Lists.List.
Require Export Crypto.Util.FixCoqMistakes.
+Require Export Crypto.Util.ZUtil.Notations.
+Require Export Crypto.Util.ZUtil.Definitions.
Import Nat.
Local Open Scope Z.
-Infix ">>" := Z.shiftr : Z_scope.
-Infix "<<" := Z.shiftl : Z_scope.
-Infix "&'" := Z.land : Z_scope.
-
Hint Extern 1 => lia : lia.
Hint Extern 1 => lra : lra.
Hint Extern 1 => nia : nia.
@@ -332,8 +330,6 @@ Module Z.
end.
Ltac peel_le := repeat peel_le_step.
- Definition pow2_mod n i := (n &' (Z.ones i)).
-
Lemma pow2_mod_spec : forall a b, (0 <= b) -> Z.pow2_mod a b = a mod (2 ^ b).
Proof.
intros.
@@ -387,7 +383,7 @@ Module Z.
else if Z_lt_dec i n then Z.testbit a i else false.
Proof.
intros; destruct (Z_lt_dec n 0); [ | apply testbit_pow2_mod; omega ].
- unfold pow2_mod.
+ unfold Z.pow2_mod.
autorewrite with Ztestbit_full;
repeat break_match;
autorewrite with Ztestbit;