aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/HTL.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/HTL.v
parentce3adde4b50ba04430a1cf0ffb0ea85168091746 (diff)
downloadvericert-f06e5fc0ee651c3ffe357c3c3302ca1517381b4c.tar.gz
vericert-f06e5fc0ee651c3ffe357c3c3302ca1517381b4c.zip
Fix warnings for Coq 8.13.2
Diffstat (limited to 'src/hls/HTL.v')
-rw-r--r--src/hls/HTL.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/hls/HTL.v b/src/hls/HTL.v
index 61ea541..8cebbfd 100644
--- a/src/hls/HTL.v
+++ b/src/hls/HTL.v
@@ -227,7 +227,7 @@ Inductive step : genv -> state -> Events.trace -> state -> Prop :=
mst = mod_st m ->
step g (Returnstate (Stackframe r m pc asr asa :: sf) i) Events.E0
(State sf m pc ((asr # mst <- (posToValue pc)) # r <- i) asa).
-Hint Constructors step : htl.
+#[export] Hint Constructors step : htl.
Inductive initial_state (p: program): state -> Prop :=
| initial_state_intro: forall b m0 m,