aboutsummaryrefslogtreecommitdiffstats
path: root/powerpc/Asm.v
diff options
context:
space:
mode:
authorBernhard Schommer <bernhardschommer@gmail.com>2015-09-03 13:22:28 +0200
committerBernhard Schommer <bernhardschommer@gmail.com>2015-09-03 13:22:28 +0200
commitc74211d87eb53cb310703dec2c504b26d7f24bdf (patch)
tree02ba6656583426df8fc43bd1d005f57326c7ea32 /powerpc/Asm.v
parent38959ad2b2d35a7d1b3479ef4298a5d754350cd8 (diff)
downloadcompcert-kvx-c74211d87eb53cb310703dec2c504b26d7f24bdf.tar.gz
compcert-kvx-c74211d87eb53cb310703dec2c504b26d7f24bdf.zip
Added builtin for mbar instruction.
This commit adds a builtin function for the mbar instruction.
Diffstat (limited to 'powerpc/Asm.v')
-rw-r--r--powerpc/Asm.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/powerpc/Asm.v b/powerpc/Asm.v
index 6444baf9..863ed6a1 100644
--- a/powerpc/Asm.v
+++ b/powerpc/Asm.v
@@ -231,6 +231,7 @@ Inductive instruction : Type :=
| Plwzx_a: ireg -> ireg -> ireg -> instruction (**r same, with 2 index regs *)
| Plwarx: ireg -> ireg -> ireg -> instruction (**r load with reservation *)
| Plwbrx: ireg -> ireg -> ireg -> instruction (**r load 32-bit int and reverse endianness *)
+ | Pmbar: int -> instruction (**r memory barrier *)
| Pmfcr: ireg -> instruction (**r move condition register to reg *)
| Pmfcrbit: ireg -> crbit -> instruction (**r move condition bit to reg (pseudo) *)
| Pmflr: ireg -> instruction (**r move LR to reg *)
@@ -898,6 +899,7 @@ Definition exec_instr (f: function) (i: instruction) (rs: regset) (m: mem) : out
| Plwsync
| Plhbrx _ _ _
| Plwzu _ _ _
+ | Pmbar _
| Pmfcr _
| Pmfspr _ _
| Pmtspr _ _