aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Reloadtyping.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/Reloadtyping.v')
-rw-r--r--backend/Reloadtyping.v6
1 files changed, 5 insertions, 1 deletions
diff --git a/backend/Reloadtyping.v b/backend/Reloadtyping.v
index 375bbfde..df0715ee 100644
--- a/backend/Reloadtyping.v
+++ b/backend/Reloadtyping.v
@@ -35,7 +35,7 @@ Require Import Reloadproof.
Hint Resolve wt_Lgetstack wt_Lsetstack wt_Lopmove
wt_Lop wt_Lload wt_Lstore wt_Lcall wt_Ltailcall
- wt_Llabel wt_Lgoto wt_Lcond wt_Lreturn: reloadty.
+ wt_Llabel wt_Lgoto wt_Lcond wt_Ljumptable wt_Lreturn: reloadty.
Remark wt_code_cons:
forall f i c, wt_instr f i -> wt_code f c -> wt_code f (i :: c).
@@ -295,6 +295,10 @@ Proof.
eauto with reloadty.
auto with reloadty.
+ assert (mreg_type (reg_for arg) = Loc.type arg).
+ eauto with reloadty.
+ auto with reloadty.
+
destruct optres; simpl in *; auto with reloadty.
apply wt_add_reload; auto with reloadty.
unfold loc_result. rewrite <- H1.