aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Cexec.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@college-de-france.fr>2019-08-02 10:41:29 +0200
committerXavier Leroy <xavierleroy@users.noreply.github.com>2019-08-05 18:33:17 +0200
commit6f737edae4b7e6243a9f11e74614f55381f62ec7 (patch)
tree9f571037b7bc16a9cd770151853876ee066069dd /cfrontend/Cexec.v
parentff1ead9fe0d816918f13e1586ecfed321f4a3bf3 (diff)
downloadcompcert-kvx-6f737edae4b7e6243a9f11e74614f55381f62ec7.tar.gz
compcert-kvx-6f737edae4b7e6243a9f11e74614f55381f62ec7.zip
Coq 8.10 compatibility: make explicit the "core" hint database
"Hint Resolve foo." becomes "Hint Resolve foo : core", or "Local Hint Resolve foo : core".
Diffstat (limited to 'cfrontend/Cexec.v')
-rw-r--r--cfrontend/Cexec.v11
1 files changed, 6 insertions, 5 deletions
diff --git a/cfrontend/Cexec.v b/cfrontend/Cexec.v
index e6bf2129..2942080b 100644
--- a/cfrontend/Cexec.v
+++ b/cfrontend/Cexec.v
@@ -1124,8 +1124,8 @@ Proof.
induction 1; intros; constructor; eauto.
Qed.
-Hint Constructors context contextlist.
-Hint Resolve context_compose contextlist_compose.
+Local Hint Constructors context contextlist : core.
+Local Hint Resolve context_compose contextlist_compose : core.
Definition reduction_ok (k: kind) (a: expr) (m: mem) (rd: reduction) : Prop :=
match k, rd with
@@ -1691,8 +1691,9 @@ Proof.
change (In (f (C0, rd)) (map f res2)). apply in_map; auto.
Qed.
-Hint Resolve reducts_incl_val reducts_incl_loc reducts_incl_listval
- reducts_incl_incontext reducts_incl_incontext2_left reducts_incl_incontext2_right.
+Local Hint Resolve reducts_incl_val reducts_incl_loc reducts_incl_listval
+ reducts_incl_incontext reducts_incl_incontext2_left
+ reducts_incl_incontext2_right : core.
Lemma step_expr_context:
forall from to C, context from to C ->
@@ -2077,7 +2078,7 @@ Ltac myinv :=
| _ => idtac
end.
-Hint Extern 3 => exact I.
+Local Hint Extern 3 => exact I : core.
Theorem do_step_sound:
forall w S rule t S',