aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Cop.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/Cop.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/Cop.v')
-rw-r--r--cfrontend/Cop.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/cfrontend/Cop.v b/cfrontend/Cop.v
index 782fb32a..aa73abb0 100644
--- a/cfrontend/Cop.v
+++ b/cfrontend/Cop.v
@@ -1131,7 +1131,7 @@ Qed.
Remark val_inject_vptrofs: forall n, Val.inject f (Vptrofs n) (Vptrofs n).
Proof. intros. unfold Vptrofs. destruct Archi.ptr64; auto. Qed.
-Hint Resolve val_inject_vtrue val_inject_vfalse val_inject_of_bool val_inject_vptrofs.
+Local Hint Resolve val_inject_vtrue val_inject_vfalse val_inject_of_bool val_inject_vptrofs : core.
Ltac TrivialInject :=
match goal with
@@ -1517,7 +1517,7 @@ Inductive val_casted: val -> type -> Prop :=
| val_casted_void: forall v,
val_casted v Tvoid.
-Hint Constructors val_casted.
+Local Hint Constructors val_casted : core.
Remark cast_int_int_idem:
forall sz sg i, cast_int_int sz sg (cast_int_int sz sg i) = cast_int_int sz sg i.