aboutsummaryrefslogtreecommitdiffstats
path: root/powerpc/Machregs.v
diff options
context:
space:
mode:
authorBernhard Schommer <bernhardschommer@gmail.com>2015-09-21 16:17:44 +0200
committerBernhard Schommer <bernhardschommer@gmail.com>2015-09-21 16:17:44 +0200
commitbc1fbdd0baaab41aa048b3214ec71bb0cc04dfcc (patch)
tree797388459aa43a97ec3cf696664540a5840839dc /powerpc/Machregs.v
parent435dc0e6fe74f0ab06737360e1dc49b42b95f1e4 (diff)
downloadcompcert-kvx-bc1fbdd0baaab41aa048b3214ec71bb0cc04dfcc.tar.gz
compcert-kvx-bc1fbdd0baaab41aa048b3214ec71bb0cc04dfcc.zip
Applied a few simplification for temporary registers.
Diffstat (limited to 'powerpc/Machregs.v')
-rw-r--r--powerpc/Machregs.v5
1 files changed, 2 insertions, 3 deletions
diff --git a/powerpc/Machregs.v b/powerpc/Machregs.v
index c464ddd6..f94c3b64 100644
--- a/powerpc/Machregs.v
+++ b/powerpc/Machregs.v
@@ -167,9 +167,8 @@ Definition builtin_atomic_compare_exchange := ident_of_string "__builtin_atomic_
Definition destroyed_by_builtin (ef: external_function): list mreg :=
match ef with
| EF_builtin id sg =>
- if ident_eq id builtin_atomic_exchange then R10::R11:: nil
- else if ident_eq id builtin_atomic_compare_exchange then R10::R11::R12:: nil
- else if ident_eq id builtin_sync_and_fetch then R3::R10::nil
+ if ident_eq id builtin_atomic_exchange then R10::nil
+ else if ident_eq id builtin_atomic_compare_exchange then R10::R11::nil
else F13 :: nil
| EF_vload _ => R11 :: nil
| EF_vstore Mint64 => R10 :: R11 :: R12 :: nil