aboutsummaryrefslogtreecommitdiffstats
path: root/aarch64/Asmgen.v
diff options
context:
space:
mode:
authorLéo Gourdin <leo.gourdin@univ-grenoble-alpes.fr>2020-11-02 17:18:56 +0100
committerLéo Gourdin <leo.gourdin@univ-grenoble-alpes.fr>2020-11-02 17:18:56 +0100
commitb4d230adb164cc1b1648ae6805c0625d6e4b7b14 (patch)
tree85ef30dcd32f2e049b7da080409d58b0e882faba /aarch64/Asmgen.v
parent241da496839a9101e843ce7b1da4a668f998498a (diff)
parent45ce514eaeb2fb1d80cb145ba769cd281195cb69 (diff)
downloadcompcert-kvx-b4d230adb164cc1b1648ae6805c0625d6e4b7b14.tar.gz
compcert-kvx-b4d230adb164cc1b1648ae6805c0625d6e4b7b14.zip
Merge branch 'aarch64_block_multiple_labels' into aarch64-postpass
Diffstat (limited to 'aarch64/Asmgen.v')
-rw-r--r--aarch64/Asmgen.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/aarch64/Asmgen.v b/aarch64/Asmgen.v
index fcc64956..33fcf34b 100644
--- a/aarch64/Asmgen.v
+++ b/aarch64/Asmgen.v
@@ -326,11 +326,11 @@ Definition unfold_bblock (bb: bblock) :=
* on the other hand could return a position pointing into the original
* basic block.
*)
- if zle (list_length_z (header bb)) 1 then
+ (*if zle (list_length_z (header bb)) 1 then*)
do bo_is <- unfold_body (body bb);
- OK (lbl ++ bo_is ++ unfold_exit (exit bb))
- else
- Error (msg "Asmgen.unfold_bblock: Multiple labels were generated.").
+ OK (lbl ++ bo_is ++ unfold_exit (exit bb)).
+ (*else*)
+ (*Error (msg "Asmgen.unfold_bblock: Multiple labels were generated.").*)
Fixpoint unfold (bbs: Asmblock.bblocks) : res Asm.code :=
match bbs with