aboutsummaryrefslogtreecommitdiffstats
path: root/aarch64/Asmgen.v
diff options
context:
space:
mode:
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 fcd12eef..d1d01a8f 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