aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asm.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-11 13:17:40 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-11 13:17:40 +0200
commit133728dcd0c9d27965b519e8b18e7bca4fd8c473 (patch)
tree4d7e2f00b985b64efffefc5b5c16bbcd10ba599d /mppa_k1c/Asm.v
parent9ff90aa440d195076a30fe4d8a055d050d84f726 (diff)
downloadcompcert-kvx-133728dcd0c9d27965b519e8b18e7bca4fd8c473.tar.gz
compcert-kvx-133728dcd0c9d27965b519e8b18e7bca4fd8c473.zip
instruction cache builtins
Diffstat (limited to 'mppa_k1c/Asm.v')
-rw-r--r--mppa_k1c/Asm.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/mppa_k1c/Asm.v b/mppa_k1c/Asm.v
index bb78eda1..b5051de3 100644
--- a/mppa_k1c/Asm.v
+++ b/mppa_k1c/Asm.v
@@ -88,6 +88,9 @@ Inductive instruction : Type :=
| Pdinval
| Pdinvall (addr: ireg)
| Pdtouchl (addr: ireg)
+ | Piinval
+ | Piinvals (addr: ireg)
+ | Pitouchl (addr: ireg)
| Pdzerol (addr: ireg)
(** Loads **)