aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Locations.v
diff options
context:
space:
mode:
authorBernhard Schommer <bernhardschommer@gmail.com>2015-09-01 09:57:01 +0200
committerBernhard Schommer <bernhardschommer@gmail.com>2015-09-01 09:57:01 +0200
commit951963b380f1ff1e0b55f8303e4ae098cedb3cb5 (patch)
tree6cc793efe8fc8d2950d7b313bfde79b2ecf40d24 /backend/Locations.v
parent7cfaf10b604372044f53cb65b03df33c23f8b26d (diff)
parent3324ece265091490d5380caf753d76aeee059d3f (diff)
downloadcompcert-951963b380f1ff1e0b55f8303e4ae098cedb3cb5.tar.gz
compcert-951963b380f1ff1e0b55f8303e4ae098cedb3cb5.zip
Merge branch 'new-builtins'
Diffstat (limited to 'backend/Locations.v')
-rw-r--r--backend/Locations.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/backend/Locations.v b/backend/Locations.v
index 5674b93a..439cd2dc 100644
--- a/backend/Locations.v
+++ b/backend/Locations.v
@@ -377,6 +377,14 @@ Module Locmap.
destruct vl; auto. destruct H. rewrite IHll; auto. apply gso; auto. apply Loc.diff_sym; auto.
Qed.
+ Fixpoint setres (res: builtin_res mreg) (v: val) (m: t) : t :=
+ match res with
+ | BR r => set (R r) v m
+ | BR_none => m
+ | BR_splitlong hi lo =>
+ setres lo (Val.loword v) (setres hi (Val.hiword v) m)
+ end.
+
End Locmap.
(** * Total ordering over locations *)