aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asmblock.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-16 19:00:55 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-16 19:00:55 +0100
commit2227019e15866870f87488630f17cbb0797d1786 (patch)
tree2a69968dc2dae750de701aab41e634690396785e /mppa_k1c/Asmblock.v
parent4e3b46ca2a30abf520672f4b1a28f91f171f6e7e (diff)
downloadcompcert-kvx-2227019e15866870f87488630f17cbb0797d1786.tar.gz
compcert-kvx-2227019e15866870f87488630f17cbb0797d1786.zip
nxor
Diffstat (limited to 'mppa_k1c/Asmblock.v')
-rw-r--r--mppa_k1c/Asmblock.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/mppa_k1c/Asmblock.v b/mppa_k1c/Asmblock.v
index 66878a94..6e55b074 100644
--- a/mppa_k1c/Asmblock.v
+++ b/mppa_k1c/Asmblock.v
@@ -342,6 +342,7 @@ Inductive arith_name_rrr : Type :=
| Porw (**r or word *)
| Pnorw (**r nor word *)
| Pxorw (**r xor word *)
+ | Pnxorw (**r nxor word *)
| Psraw (**r shift right arithmetic word *)
| Psrlw (**r shift right logical word *)
| Psllw (**r shift left logical word *)
@@ -373,6 +374,7 @@ Inductive arith_name_rri32 : Type :=
| Poriw (**r or imm word *)
| Pnoriw (**r nor imm word *)
| Pxoriw (**r xor imm word *)
+ | Pnxoriw (**r nxor imm word *)
| Psraiw (**r shift right arithmetic imm word *)
| Psrliw (**r shift right logical imm word *)
| Pslliw (**r shift left logical imm word *)
@@ -1099,6 +1101,7 @@ Definition arith_eval_rrr n v1 v2 :=
| Porw => Val.or v1 v2
| Pnorw => Val.notint (Val.or v1 v2)
| Pxorw => Val.xor v1 v2
+ | Pnxorw => Val.notint (Val.xor v1 v2)
| Psrlw => Val.shru v1 v2
| Psraw => Val.shr v1 v2
| Psllw => Val.shl v1 v2
@@ -1130,6 +1133,7 @@ Definition arith_eval_rri32 n v i :=
| Poriw => Val.or v (Vint i)
| Pnoriw => Val.notint (Val.or v (Vint i))
| Pxoriw => Val.xor v (Vint i)
+ | Pnxoriw => Val.notint (Val.xor v (Vint i))
| Psraiw => Val.shr v (Vint i)
| Psrliw => Val.shru v (Vint i)
| Pslliw => Val.shl v (Vint i)