aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Constprop.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@inria.fr>2017-06-16 11:53:28 +0200
committerBernhard Schommer <bschommer@users.noreply.github.com>2017-07-06 15:41:51 +0200
commit2ff53c2361773f28027ccc8332e1830686d5bbc6 (patch)
tree2c0b1dc7201bd3618859cc5dc2257dbf07e996de /backend/Constprop.v
parentdff22ef6d855973e0e0f05c7203a6bfa9a4cf01a (diff)
downloadcompcert-kvx-2ff53c2361773f28027ccc8332e1830686d5bbc6.tar.gz
compcert-kvx-2ff53c2361773f28027ccc8332e1830686d5bbc6.zip
Extend builtin arguments with a pointer addition operator, continued
- Add support for PowerPC, with all addressing modes. - Add support for ARM, with "reg + ofs" addressing mode. - Add support for RISC-V, with the one addressing mode. - Constprop.v: forgot to recurse in BA_addptr - volatile4 test: more tests
Diffstat (limited to 'backend/Constprop.v')
-rw-r--r--backend/Constprop.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/backend/Constprop.v b/backend/Constprop.v
index 151f8418..d8211ffe 100644
--- a/backend/Constprop.v
+++ b/backend/Constprop.v
@@ -98,6 +98,8 @@ Fixpoint builtin_arg_reduction (ae: AE.t) (a: builtin_arg reg) :=
| BA_int nhi, BA_int nlo => BA_long (Int64.ofwords nhi nlo)
| hi', lo' => BA_splitlong hi' lo'
end
+ | BA_addptr a1 a2 =>
+ BA_addptr (builtin_arg_reduction ae a1) (builtin_arg_reduction ae a2)
| _ => a
end.