aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/HTL.v
diff options
context:
space:
mode:
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 ce7d37e..f16aef5 100644
--- a/src/hls/HTL.v
+++ b/src/hls/HTL.v
@@ -318,7 +318,7 @@ Inductive step : genv -> state -> Events.trace -> state -> Prop :=
(State sf mid m st (asr # fin <- (ZToValue 0)) asa).
-Hint Constructors step : htl.
+#[export] Hint Constructors step : htl.
Inductive initial_state (p: program): state -> Prop :=
| initial_state_intro: forall b m0 m,