aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/ValueInt.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2020-11-26 01:00:13 +0000
committerYann Herklotz <git@yannherklotz.com>2020-11-26 01:00:13 +0000
commit29bee524cccfe08c680f655b1969a4c421e0a969 (patch)
tree9a98159b31f566ad48712b7ada8bb6c25cf763c5 /src/hls/ValueInt.v
parentd64f47def97420f40f61a53c385143b94b30b5b3 (diff)
downloadvericert-29bee524cccfe08c680f655b1969a4c421e0a969.tar.gz
vericert-29bee524cccfe08c680f655b1969a4c421e0a969.zip
Fix build for Coq 8.12.1
Diffstat (limited to 'src/hls/ValueInt.v')
-rw-r--r--src/hls/ValueInt.v10
1 files changed, 0 insertions, 10 deletions
diff --git a/src/hls/ValueInt.v b/src/hls/ValueInt.v
index f1fd056..e434abc 100644
--- a/src/hls/ValueInt.v
+++ b/src/hls/ValueInt.v
@@ -17,8 +17,6 @@
*)
(* begin hide *)
-From bbv Require Import Word.
-From bbv Require HexNotation WordScope.
From Coq Require Import ZArith.ZArith FSets.FMapPositive Lia.
From compcert Require Import lib.Integers common.Values.
From vericert Require Import Vericertlib.
@@ -98,14 +96,6 @@ Definition boolToValue (b : bool) : value :=
(** ** Arithmetic operations *)
-Definition unify_word (sz1 sz2 : nat) (w1 : word sz2): sz1 = sz2 -> word sz1.
-intros; subst; assumption. Defined.
-
-Lemma unify_word_unfold :
- forall sz w,
- unify_word sz sz w eq_refl = w.
-Proof. auto. Qed.
-
Inductive val_value_lessdef: val -> value -> Prop :=
| val_value_lessdef_int:
forall i v',