aboutsummaryrefslogtreecommitdiffstats
path: root/aarch64/Asmblock.v
diff options
context:
space:
mode:
authorJustus Fasse <justus.fasse@etu.univ-grenoble-alpes.fr>2020-07-13 17:43:22 +0200
committerJustus Fasse <justus.fasse@etu.univ-grenoble-alpes.fr>2020-07-13 17:43:22 +0200
commitc48fd3f91f6dc9a35c7c9cb4a4b21d0598d91930 (patch)
tree2822f759f10a1173329f255ad80a8208084ecb93 /aarch64/Asmblock.v
parent45049f8a085bb916009ee9154d7218a1a287c0da (diff)
downloadcompcert-kvx-c48fd3f91f6dc9a35c7c9cb4a4b21d0598d91930.tar.gz
compcert-kvx-c48fd3f91f6dc9a35c7c9cb4a4b21d0598d91930.zip
Generate both Pcsel and Pfsel
In Asmblock, Pcsel is used for both integer and floating-point conditional selection. A previous commit (c764ff84) had incorrectly reverted the merging of Pfsel into Pcsel.
Diffstat (limited to 'aarch64/Asmblock.v')
-rw-r--r--aarch64/Asmblock.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/aarch64/Asmblock.v b/aarch64/Asmblock.v
index e362753b..ba6a64fa 100644
--- a/aarch64/Asmblock.v
+++ b/aarch64/Asmblock.v
@@ -445,7 +445,7 @@ Inductive ar_instruction : Type :=
(* PArithFR0 *)
| Pfmovi (fsz : fsize) (rd : freg) (r1 : ireg0) (**r copy int reg to FP reg *)
(* PArithCPPP *)
- | Pcsel (rd r1 r2 : ireg) (c : testcond) (**r int/float conditional move *)
+ | Pcsel (rd r1 r2 : preg) (c : testcond) (**r int/float conditional move *)
(* PArithAFFF *)
| Pfnmul (fsz : fsize) (rd r1 r2 : freg) (**r multiply-negate *)
.