aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asm.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-11 09:28:59 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-11 09:28:59 +0200
commitcdb5ec57d700c5409c0717bb99258a5effed9601 (patch)
tree18d02787dda85ce6eb3f2904bd964c6ab29be50b /mppa_k1c/Asm.v
parent466767d23cbc816b5787e6768e5f9a98a95abca9 (diff)
downloadcompcert-kvx-cdb5ec57d700c5409c0717bb99258a5effed9601.tar.gz
compcert-kvx-cdb5ec57d700c5409c0717bb99258a5effed9601.zip
wfxl / wfxm
Diffstat (limited to 'mppa_k1c/Asm.v')
-rw-r--r--mppa_k1c/Asm.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/mppa_k1c/Asm.v b/mppa_k1c/Asm.v
index 7c6bd013..9517099c 100644
--- a/mppa_k1c/Asm.v
+++ b/mppa_k1c/Asm.v
@@ -76,6 +76,8 @@ Inductive instruction : Type :=
| Ploopdo (count: ireg) (loopend: label)
| Pgetn (n: int) (dst: ireg)
| Psetn (n: int) (src: ireg)
+ | Pwfxl (n: int) (src: ireg)
+ | Pwfxm (n: int) (src: ireg)
(** Loads **)
| Plb (rd: ireg) (ra: ireg) (ofs: addressing) (**r load byte *)