aboutsummaryrefslogtreecommitdiffstats
path: root/arm
diff options
context:
space:
mode:
Diffstat (limited to 'arm')
-rw-r--r--arm/Asmexpand.ml4
-rw-r--r--arm/Asmgenproof1.v4
2 files changed, 4 insertions, 4 deletions
diff --git a/arm/Asmexpand.ml b/arm/Asmexpand.ml
index 629d0fcc..b81ae74b 100644
--- a/arm/Asmexpand.ml
+++ b/arm/Asmexpand.ml
@@ -111,8 +111,8 @@ let memcpy_small_arg sz arg tmp =
assert false
let expand_builtin_memcpy_small sz al src dst =
- let (tsrc, tdst) =
- if dst <> BA (IR IR2) then (IR2, IR3) else (IR3, IR2) in
+ let tsrc = if dst <> BA (IR IR2) then IR2 else IR3 in
+ let tdst = if src <> BA (IR IR3) then IR3 else IR2 in
let (rsrc, osrc) = memcpy_small_arg sz src tsrc in
let (rdst, odst) = memcpy_small_arg sz dst tdst in
let rec copy osrc odst sz =
diff --git a/arm/Asmgenproof1.v b/arm/Asmgenproof1.v
index 7a707f32..729ddb4f 100644
--- a/arm/Asmgenproof1.v
+++ b/arm/Asmgenproof1.v
@@ -1218,7 +1218,7 @@ Proof.
split. unfold rs2; Simpl. unfold rs1; Simpl.
unfold Val.shr, Val.shl; destruct (rs x0); auto.
change (Int.ltu (Int.repr 24) Int.iwordsize) with true; simpl.
- f_equal. symmetry. apply (Int.sign_ext_shr_shl 8). compute; auto.
+ f_equal. symmetry. apply (Int.sign_ext_shr_shl 8). compute; intuition congruence.
intros. unfold rs2, rs1; Simpl.
(* Ocast16signed *)
destruct Archi.thumb2_support.
@@ -1231,7 +1231,7 @@ Proof.
split. unfold rs2; Simpl. unfold rs1; Simpl.
unfold Val.shr, Val.shl; destruct (rs x0); auto.
change (Int.ltu (Int.repr 16) Int.iwordsize) with true; simpl.
- f_equal. symmetry. apply (Int.sign_ext_shr_shl 16). compute; auto.
+ f_equal. symmetry. apply (Int.sign_ext_shr_shl 16). compute; intuition congruence.
intros. unfold rs2, rs1; Simpl.
(* Oaddimm *)
generalize (addimm_correct x x0 i k rs m).