aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/HTLgen.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2021-10-09 14:30:03 +0100
committerYann Herklotz <git@yannherklotz.com>2021-10-09 14:30:03 +0100
commitf06e5fc0ee651c3ffe357c3c3302ca1517381b4c (patch)
tree15821bec5295bc84b95bd44b00e0d192c58c36fe /src/hls/HTLgen.v
parentce3adde4b50ba04430a1cf0ffb0ea85168091746 (diff)
downloadvericert-f06e5fc0ee651c3ffe357c3c3302ca1517381b4c.tar.gz
vericert-f06e5fc0ee651c3ffe357c3c3302ca1517381b4c.zip
Fix warnings for Coq 8.13.2
Diffstat (limited to 'src/hls/HTLgen.v')
-rw-r--r--src/hls/HTLgen.v14
1 files changed, 7 insertions, 7 deletions
diff --git a/src/hls/HTLgen.v b/src/hls/HTLgen.v
index 4d60a24..3f4e513 100644
--- a/src/hls/HTLgen.v
+++ b/src/hls/HTLgen.v
@@ -33,11 +33,11 @@ Require Import vericert.hls.HTL.
Require Import vericert.hls.ValueInt.
Require Import vericert.hls.Verilog.
-Hint Resolve AssocMap.gempty : htlh.
-Hint Resolve AssocMap.gso : htlh.
-Hint Resolve AssocMap.gss : htlh.
-Hint Resolve Ple_refl : htlh.
-Hint Resolve Ple_succ : htlh.
+#[local] Hint Resolve AssocMap.gempty : htlh.
+#[local] Hint Resolve AssocMap.gso : htlh.
+#[local] Hint Resolve AssocMap.gss : htlh.
+#[local] Hint Resolve Ple_refl : htlh.
+#[local] Hint Resolve Ple_succ : htlh.
Record state: Type := mkstate {
st_st : reg;
@@ -74,10 +74,10 @@ Module HTLState <: State.
s1.(st_controllogic)!n = None
\/ s2.(st_controllogic)!n = s1.(st_controllogic)!n) ->
st_incr s1 s2.
- Hint Constructors st_incr : htlh.
+ #[export] Hint Constructors st_incr : htlh.
Definition st_prop := st_incr.
- Hint Unfold st_prop : htlh.
+ #[export] Hint Unfold st_prop : htlh.
Lemma st_refl : forall s, st_prop s s. Proof. auto with htlh. Qed.