aboutsummaryrefslogtreecommitdiffstats
path: root/powerpc/Asm.v
diff options
context:
space:
mode:
authorBernhard Schommer <bernhardschommer@gmail.com>2015-08-17 16:11:47 +0200
committerBernhard Schommer <bernhardschommer@gmail.com>2015-08-17 16:11:47 +0200
commit7fe3c745283dcfd7cd304bca68ae2cc3ea7cd4a5 (patch)
treef9e3d36e7c1c08c8dd4d95118d268fdfa1c1244b /powerpc/Asm.v
parent2c2fca9756e38535db7697c6f53126003b624c6c (diff)
downloadcompcert-kvx-7fe3c745283dcfd7cd304bca68ae2cc3ea7cd4a5.tar.gz
compcert-kvx-7fe3c745283dcfd7cd304bca68ae2cc3ea7cd4a5.zip
Added builtin for the dcbf 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 f1e84146..b7656dc4 100644
--- a/powerpc/Asm.v
+++ b/powerpc/Asm.v
@@ -165,6 +165,7 @@ Inductive instruction : Type :=
| Pcreqv: crbit -> crbit -> crbit -> instruction (**r not-xor between condition bits *)
| Pcror: crbit -> crbit -> crbit -> instruction (**r or between condition bits *)
| Pcrxor: crbit -> crbit -> crbit -> instruction (**r xor between condition bits *)
+ | Pdcbf: ireg -> ireg -> instruction (**r data cache flush *)
| Pdcbi: ireg -> ireg -> instruction (**r data cache invalidate *)
| Pdivw: ireg -> ireg -> ireg -> instruction (**r signed division *)
| Pdivwu: ireg -> ireg -> ireg -> instruction (**r unsigned division *)
@@ -859,6 +860,7 @@ Definition exec_instr (f: function) (i: instruction) (rs: regset) (m: mem) : out
| Pcntlzw _ _
| Pcreqv _ _ _
| Pcrxor _ _ _
+ | Pdcbf _ _
| Pdcbi _ _
| Peieio
| Pfctiw _ _