From 3fd5f652ba38a0b308b6e2e86783d82b861fb5bf Mon Sep 17 00:00:00 2001 From: Samuel Gruetter Date: Fri, 2 Feb 2018 16:09:01 -0500 Subject: minor updates needed to make it compile with bbv removing lemma wordToNat_wzero is ok because it's already in bbv --- src/Util/WordUtil.v | 11 ++--------- 1 file changed, 2 insertions(+), 9 deletions(-) (limited to 'src/Util/WordUtil.v') diff --git a/src/Util/WordUtil.v b/src/Util/WordUtil.v index 64cfda434..c1eeb138b 100644 --- a/src/Util/WordUtil.v +++ b/src/Util/WordUtil.v @@ -15,8 +15,8 @@ Require Import Crypto.Util.Tactics.DestructHead. Require Import Crypto.Util.Tactics.RewriteHyp. Require Import Crypto.Util.Sigma. -Require Import Bedrock.Word. -Require Import Bedrock.Nomega. +Require Import bbv.WordScope. +Require Import bbv.Nomega. Require Import Crypto.Util.FixCoqMistakes. @@ -370,8 +370,6 @@ Section WordToN. + clear IHk'. shatter x; simpl. - rewrite N.succ_double_spec; simpl. - rewrite kill_match. replace (N.pos (Pos.of_succ_nat k')) with (N.succ (N.of_nat k')) @@ -826,11 +824,6 @@ Definition setbit {b} n {H:n < b} (w:word b) : word b := Definition clearbit {b} n {H:n < b} (w:word b) : word b := wand (cast_word( wones n ++ wzero 1 ++ wones (b-n-1) )) w. -Lemma wordToNat_wzero {n} : wordToNat (wzero n) = 0. -Proof. - unfold wzero; induction n as [|n IHn]; simpl; try rewrite_hyp!*; omega. -Qed. - Lemma wordToNat_combine : forall {a} (wa:word a) {b} (wb:word b), wordToNat (wa ++ wb) = wordToNat wa + 2^a * wordToNat wb. Proof. -- cgit v1.2.3