aboutsummaryrefslogtreecommitdiffstats
path: root/powerpc/Asm.v
diff options
context:
space:
mode:
authorBernhard Schommer <bernhardschommer@gmail.com>2015-09-02 17:17:00 +0200
committerBernhard Schommer <bernhardschommer@gmail.com>2015-09-02 17:17:00 +0200
commitcfee340dc514e2cfbc5df910f7aa687e78a54d41 (patch)
tree1b6544f0dbbc628ee1b10c191a794c1ef5ab9ab8 /powerpc/Asm.v
parent30ebbcd0731f680d1d283afb99318fb9d6e9cead (diff)
downloadcompcert-kvx-cfee340dc514e2cfbc5df910f7aa687e78a54d41.tar.gz
compcert-kvx-cfee340dc514e2cfbc5df910f7aa687e78a54d41.zip
Added builtin for the icbtls instruction.
This commit adds a builtin for the icbtls 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 43ddc1ed..32c7ba70 100644
--- a/powerpc/Asm.v
+++ b/powerpc/Asm.v
@@ -207,6 +207,7 @@ Inductive instruction : Type :=
| Pfsel: freg -> freg -> freg -> freg -> instruction (**r FP conditional move *)
| Pisync: instruction (**r ISYNC barrier *)
| Picbi: ireg -> ireg -> instruction (**r instruction cache invalidate *)
+ | Picbtls: int -> ireg -> instruction (**r instruction cache block touch and lock set *)
| Plbz: ireg -> constant -> ireg -> instruction (**r load 8-bit unsigned int *)
| Plbzx: ireg -> ireg -> ireg -> instruction (**r same, with 2 index regs *)
| Plfd: freg -> constant -> ireg -> instruction (**r load 64-bit float *)
@@ -890,6 +891,7 @@ Definition exec_instr (f: function) (i: instruction) (rs: regset) (m: mem) : out
| Plwarx _ _ _
| Plwbrx _ _ _
| Picbi _ _
+ | Picbtls _ _
| Pisync
| Plwsync
| Plhbrx _ _ _