aboutsummaryrefslogtreecommitdiffstats
path: root/common/Events.v
diff options
context:
space:
mode:
Diffstat (limited to 'common/Events.v')
-rw-r--r--common/Events.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/common/Events.v b/common/Events.v
index 0ada1207..2e076523 100644
--- a/common/Events.v
+++ b/common/Events.v
@@ -27,6 +27,9 @@ Require Import Memory.
Require Import Globalenvs.
Require Import Builtins.
+(** Backwards compatibility for Hint Rewrite locality attributes. *)
+Set Warnings "-unsupported-attributes".
+
(** * Events and traces *)
(** The observable behaviour of programs is stated in terms of
@@ -113,6 +116,7 @@ Proof.
induction t1; intros; simpl. auto. decEq; auto.
Qed.
+#[global]
Hint Rewrite E0_left E0_right Eapp_assoc
E0_left_inf Eappinf_assoc: trace_rewrite.