aboutsummaryrefslogtreecommitdiffstats
path: root/aarch64/Asm.v
diff options
context:
space:
mode:
authorJustus Fasse <justus.fasse@etu.univ-grenoble-alpes.fr>2020-07-20 11:47:06 +0200
committerJustus Fasse <justus.fasse@etu.univ-grenoble-alpes.fr>2020-07-21 17:41:40 +0200
commit61410a182bfeb82043c1cb519b81d3dc8f4e997e (patch)
tree3f4ed4a808ec647a37e2c3d9d4d124948bebae54 /aarch64/Asm.v
parent1674f32a0339a0801489336ec15a2e116ba4f95b (diff)
downloadcompcert-kvx-61410a182bfeb82043c1cb519b81d3dc8f4e997e.tar.gz
compcert-kvx-61410a182bfeb82043c1cb519b81d3dc8f4e997e.zip
Add dynamically checked assumption to simplify Asmgenproof
Previously Asmblock.label_pos and Asm.label_pos could point to different memory location for the same label.
Diffstat (limited to 'aarch64/Asm.v')
-rw-r--r--aarch64/Asm.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/aarch64/Asm.v b/aarch64/Asm.v
index 369e6f3b..dc1faddd 100644
--- a/aarch64/Asm.v
+++ b/aarch64/Asm.v
@@ -240,7 +240,7 @@ Fixpoint label_pos (lbl: label) (pos: Z) (c: code) {struct c} : option Z :=
match c with
| nil => None
| instr :: c' =>
- if is_label lbl instr then Some (pos + 1) else label_pos lbl (pos + 1) c'
+ if is_label lbl instr then Some pos else label_pos lbl (pos + 1) c'
end.
Definition nextinstr (rs: regset) :=