aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asmblock.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-18 22:08:45 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-18 22:08:45 +0100
commitddbe4221279f9e75b4ed075156420e62a92f28d9 (patch)
treedec89af696277d93761f53a7d71de7cb7f1b7fbc /mppa_k1c/Asmblock.v
parentea12bb63c4ff63c12a383b8b66dff11fc5dc6e65 (diff)
downloadcompcert-kvx-ddbe4221279f9e75b4ed075156420e62a92f28d9.tar.gz
compcert-kvx-ddbe4221279f9e75b4ed075156420e62a92f28d9.zip
maddw dans la génération
Diffstat (limited to 'mppa_k1c/Asmblock.v')
-rw-r--r--mppa_k1c/Asmblock.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/mppa_k1c/Asmblock.v b/mppa_k1c/Asmblock.v
index 9b51ea33..b3e1532d 100644
--- a/mppa_k1c/Asmblock.v
+++ b/mppa_k1c/Asmblock.v
@@ -443,6 +443,9 @@ Coercion PArithRF64: arith_name_rf64 >-> Funclass.
Coercion PArithRRR: arith_name_rrr >-> Funclass.
Coercion PArithRRI32: arith_name_rri32 >-> Funclass.
Coercion PArithRRI64: arith_name_rri64 >-> Funclass.
+Coercion PArithARRR: arith_name_arrr >-> Funclass.
+Coercion PArithARRI32: arith_name_arri32 >-> Funclass.
+Coercion PArithARRI64: arith_name_arri64 >-> Funclass.
Inductive basic : Type :=
| PArith (i: ar_instruction)