aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asm.v
diff options
context:
space:
mode:
authorCyril SIX <cyril.six@kalray.eu>2019-03-19 15:50:22 +0100
committerCyril SIX <cyril.six@kalray.eu>2019-03-19 15:50:22 +0100
commitf321f75979d18ab99f226b2c5d6bbb59bffb5cac (patch)
tree54dfd0c7ce3a0569549120c786026b6b33431254 /mppa_k1c/Asm.v
parentb169a1c8b88feee186d96c107562aff847caf235 (diff)
downloadcompcert-kvx-f321f75979d18ab99f226b2c5d6bbb59bffb5cac.tar.gz
compcert-kvx-f321f75979d18ab99f226b2c5d6bbb59bffb5cac.zip
Pseudo instruction for 32 bits division, no code generation yet
Diffstat (limited to 'mppa_k1c/Asm.v')
-rw-r--r--mppa_k1c/Asm.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/mppa_k1c/Asm.v b/mppa_k1c/Asm.v
index 8486e25d..029ac995 100644
--- a/mppa_k1c/Asm.v
+++ b/mppa_k1c/Asm.v
@@ -50,6 +50,9 @@ Inductive instruction : Type :=
| Psemi (**r semi colon separating bundles *)
| Pnop (**r instruction that does nothing *)
+ | Pdiv (**r 32 bits integer division *)
+ | Pdivu (**r 32 bits integer division *)
+
(** builtins *)
| Pclzll (rd rs: ireg)
| Pstsud (rd rs1 rs2: ireg)
@@ -209,6 +212,8 @@ Inductive instruction : Type :=
Definition control_to_instruction (c: control) :=
match c with
| PExpand (Asmblock.Pbuiltin ef args res) => Pbuiltin ef args res
+ | PExpand (Asmblock.Pdiv) => Pdiv
+ | PExpand (Asmblock.Pdivu) => Pdivu
| PCtlFlow Asmblock.Pret => Pret
| PCtlFlow (Asmblock.Pcall l) => Pcall l
| PCtlFlow (Asmblock.Picall r) => Picall r