aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asm.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-11 13:11:13 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-11 13:11:13 +0200
commit9ff90aa440d195076a30fe4d8a055d050d84f726 (patch)
tree415d9145ff9414b47370ac86c7c221fda694d628 /mppa_k1c/Asm.v
parent71bfa128316019b0199db87acdf31deb9f9e7405 (diff)
downloadcompcert-kvx-9ff90aa440d195076a30fe4d8a055d050d84f726.tar.gz
compcert-kvx-9ff90aa440d195076a30fe4d8a055d050d84f726.zip
data cache builtins
Diffstat (limited to 'mppa_k1c/Asm.v')
-rw-r--r--mppa_k1c/Asm.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/mppa_k1c/Asm.v b/mppa_k1c/Asm.v
index 55138a3f..bb78eda1 100644
--- a/mppa_k1c/Asm.v
+++ b/mppa_k1c/Asm.v
@@ -85,6 +85,10 @@ Inductive instruction : Type :=
| Pstop
| Pbarrier
| Pfence
+ | Pdinval
+ | Pdinvall (addr: ireg)
+ | Pdtouchl (addr: ireg)
+ | Pdzerol (addr: ireg)
(** Loads **)
| Plb (rd: ireg) (ra: ireg) (ofs: addressing) (**r load byte *)