aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asm.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-10 22:50:06 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-10 22:50:06 +0200
commit7cc001e63990ae5e8cf2f75b5148093e31fbdc85 (patch)
tree2bc8e68ebe99c4b2d169e713b8f805eb1f34c2c4 /mppa_k1c/Asm.v
parent84d6fd30d9cbf684fa14d2f54c23ef582b298eb0 (diff)
downloadcompcert-kvx-7cc001e63990ae5e8cf2f75b5148093e31fbdc85.tar.gz
compcert-kvx-7cc001e63990ae5e8cf2f75b5148093e31fbdc85.zip
get / set k1
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 303a624c..7c6bd013 100644
--- a/mppa_k1c/Asm.v
+++ b/mppa_k1c/Asm.v
@@ -72,7 +72,10 @@ Inductive instruction : Type :=
| Pcb (bt: btest) (r: ireg) (l: label) (**r branch based on btest *)
| Pcbu (bt: btest) (r: ireg) (l: label) (**r branch based on btest with unsigned semantics *)
| Pjumptable (r: ireg) (labels: list label)
+
| Ploopdo (count: ireg) (loopend: label)
+ | Pgetn (n: int) (dst: ireg)
+ | Psetn (n: int) (src: ireg)
(** Loads **)
| Plb (rd: ireg) (ra: ireg) (ofs: addressing) (**r load byte *)