aboutsummaryrefslogtreecommitdiffstats
path: root/aarch64/Asmgen.v
diff options
context:
space:
mode:
authorLéo Gourdin <leo.gourdin@univ-grenoble-alpes.fr>2020-11-01 13:02:25 +0100
committerLéo Gourdin <leo.gourdin@univ-grenoble-alpes.fr>2020-11-01 13:02:25 +0100
commit45ce514eaeb2fb1d80cb145ba769cd281195cb69 (patch)
treea48b9b24e8dbd92afa7ced634fc3becdd10d1c81 /aarch64/Asmgen.v
parent8de1a1f5811470bc1d7d1a7b2f0e5193de40698e (diff)
downloadcompcert-kvx-45ce514eaeb2fb1d80cb145ba769cd281195cb69.tar.gz
compcert-kvx-45ce514eaeb2fb1d80cb145ba769cd281195cb69.zip
Yarpgen C file to test multiple labels and corresponding code
In this branch I remove the multiple label limitation to pass some tests but the proof is admitted !
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