aboutsummaryrefslogtreecommitdiffstats
path: root/powerpc/Asm.v
diff options
context:
space:
mode:
authorMichael Schmidt <github@mschmidt.me>2015-12-15 09:17:07 +0100
committerMichael Schmidt <github@mschmidt.me>2015-12-15 09:17:07 +0100
commit91029ac1749b8186c17c6cb14347066be8226434 (patch)
treec4c1670c20a2cc12dfa08402a91e04e85fe45f74 /powerpc/Asm.v
parent67fda21314a577d6ae2bc9a5abf6df329b8ba85a (diff)
downloadcompcert-kvx-91029ac1749b8186c17c6cb14347066be8226434.tar.gz
compcert-kvx-91029ac1749b8186c17c6cb14347066be8226434.zip
Bug 17752, add rldicr instruction for PowerPC
Diffstat (limited to 'powerpc/Asm.v')
-rw-r--r--powerpc/Asm.v4
1 files changed, 3 insertions, 1 deletions
diff --git a/powerpc/Asm.v b/powerpc/Asm.v
index 228977c2..a9b60fbd 100644
--- a/powerpc/Asm.v
+++ b/powerpc/Asm.v
@@ -259,6 +259,7 @@ Inductive instruction : Type :=
| Pori: ireg -> ireg -> constant -> instruction (**r or with immediate *)
| Poris: ireg -> ireg -> constant -> instruction (**r or with immediate high *)
| Prldicl: ireg -> ireg -> int -> int -> instruction (**r rotate and mask left (PPC64) *)
+ | Prldicr: ireg -> ireg -> int -> int -> instruction (**r rotate and mask right (PPC64) *)
| Prlwinm: ireg -> ireg -> int -> int -> instruction (**r rotate and mask *)
| Prlwimi: ireg -> ireg -> int -> int -> instruction (**r rotate and insert *)
| Pslw: ireg -> ireg -> ireg -> instruction (**r shift left *)
@@ -267,7 +268,7 @@ Inductive instruction : Type :=
| Psrw: ireg -> ireg -> ireg -> instruction (**r shift right unsigned *)
| Pstb: ireg -> constant -> ireg -> instruction (**r store 8-bit int *)
| Pstbx: ireg -> ireg -> ireg -> instruction (**r same, with 2 index regs *)
- | Pstdu: ireg -> constant -> ireg -> instruction (**r store 64-bit integer with update (PPC64) *)
+ | Pstdu: ireg -> constant -> ireg -> instruction (**r store 64-bit integer with update (PPC64) *)
| Pstfd: freg -> constant -> ireg -> instruction (**r store 64-bit float *)
| Pstfdu: freg -> constant -> ireg -> instruction (**r store 64-bit float with update *)
| Pstfdx: freg -> ireg -> ireg -> instruction (**r same, with 2 index regs *)
@@ -925,6 +926,7 @@ Definition exec_instr (f: function) (i: instruction) (rs: regset) (m: mem) : out
| Pmfspr _ _
| Pmtspr _ _
| Prldicl _ _ _ _
+ | Prldicr _ _ _ _
| Pstdu _ _ _
| Pstwbrx _ _ _
| Pstwcx_ _ _ _