aboutsummaryrefslogtreecommitdiffstats
path: root/aarch64/Op.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-10-19 18:20:28 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-10-19 18:20:28 +0200
commit1deadbf2715e435f2599c415c629ad0f042d40a6 (patch)
tree087db464b7d4aef1c8d140c68542755b524145db /aarch64/Op.v
parent996a2e5bbc4826d95144b62f5218b6e3e1e7d881 (diff)
downloadcompcert-kvx-1deadbf2715e435f2599c415c629ad0f042d40a6.tar.gz
compcert-kvx-1deadbf2715e435f2599c415c629ad0f042d40a6.zip
op_valid_pointer_eq for aarch64
Diffstat (limited to 'aarch64/Op.v')
-rw-r--r--aarch64/Op.v14
1 files changed, 14 insertions, 0 deletions
diff --git a/aarch64/Op.v b/aarch64/Op.v
index 0a29ff3e..f2a8e6fb 100644
--- a/aarch64/Op.v
+++ b/aarch64/Op.v
@@ -1202,6 +1202,20 @@ Proof.
rewrite (cond_depends_on_memory_correct cond args m1 m2 H). auto.
Qed.
+Lemma op_valid_pointer_eq:
+ forall (F V: Type) (ge: Genv.t F V) sp op args m1 m2,
+ (forall b z, Mem.valid_pointer m1 b z = Mem.valid_pointer m2 b z) ->
+ eval_operation ge sp op args m1 = eval_operation ge sp op args m2.
+Proof.
+ intros until m2. destruct op eqn:OP; simpl; try congruence.
+ - intros MEM; destruct cond; simpl; try congruence;
+ repeat (destruct args; simpl; try congruence);
+ erewrite cmpu_bool_valid_pointer_eq || erewrite cmplu_bool_valid_pointer_eq; eauto.
+ - intro MEM; destruct cond; simpl; try congruence;
+ repeat (destruct args; simpl; try congruence);
+ erewrite cmpu_bool_valid_pointer_eq || erewrite cmplu_bool_valid_pointer_eq; eauto.
+Qed.
+
(** Global variables mentioned in an operation or addressing mode *)
Definition globals_addressing (addr: addressing) : list ident :=