aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Lineartyping.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@inria.fr>2015-08-21 11:05:36 +0200
committerXavier Leroy <xavier.leroy@inria.fr>2015-08-21 11:05:36 +0200
commit54f97d1988f623ba7422e13a504caeb5701ba93c (patch)
treed8dea46837352979490f4ed4516f9649fef41b98 /backend/Lineartyping.v
parentb4846ffadfa3fbb73ffa7d9c43e5218adeece8da (diff)
downloadcompcert-kvx-54f97d1988f623ba7422e13a504caeb5701ba93c.tar.gz
compcert-kvx-54f97d1988f623ba7422e13a504caeb5701ba93c.zip
Refactoring of builtins and annotations in the back-end.
Before, the back-end languages had distinct instructions - Iannot for annotations, taking structured expressions (annot_arg) as arguments, and producing no results' - Ibuiltin for other builtins, using simple pseudoregs/locations/registers as arguments and results. This branch enriches Ibuiltin instructions so that they take structured expressions (builtin_arg and builtin_res) as arguments and results. This way, - Annotations fit the general pattern of builtin functions, so Iannot instructions are removed. - EF_vload_global and EF_vstore_global become useless, as the same optimization can be achieved by EF_vload/vstore taking a structured argument of the "address of global" kind. - Better code can be generated for builtin_memcpy between stack locations, or volatile accesses to stack locations. Finally, this commit also introduces a new kind of external function, EF_debug, which is like EF_annot but produces no observable events. It will be used later to transport debug info through the back-end, without preventing optimizations.
Diffstat (limited to 'backend/Lineartyping.v')
-rw-r--r--backend/Lineartyping.v40
1 files changed, 28 insertions, 12 deletions
diff --git a/backend/Lineartyping.v b/backend/Lineartyping.v
index c093b62d..2c8de98e 100644
--- a/backend/Lineartyping.v
+++ b/backend/Lineartyping.v
@@ -55,6 +55,13 @@ Definition loc_valid (l: loc) : bool :=
| S _ _ _ => false
end.
+Fixpoint wt_builtin_res (ty: typ) (res: builtin_res mreg) : bool :=
+ match res with
+ | BR r => subtype ty (mreg_type r)
+ | BR_none => true
+ | BR_longofwords hi lo => wt_builtin_res Tint hi && wt_builtin_res Tint lo
+ end.
+
Definition wt_instr (i: instruction) : bool :=
match i with
| Lgetstack sl ofs ty r =>
@@ -74,9 +81,8 @@ Definition wt_instr (i: instruction) : bool :=
| Ltailcall sg ros =>
zeq (size_arguments sg) 0
| Lbuiltin ef args res =>
- subtype_list (proj_sig_res' (ef_sig ef)) (map mreg_type res)
- | Lannot ef args =>
- forallb loc_valid (params_of_annot_args args)
+ wt_builtin_res (proj_sig_res (ef_sig ef)) res
+ && forallb loc_valid (params_of_builtin_args args)
| _ =>
true
end.
@@ -161,6 +167,20 @@ Proof.
destruct H. apply IHvl; auto. apply wt_setreg; auto.
Qed.
+Lemma wt_setres:
+ forall res ty v rs,
+ wt_builtin_res ty res = true ->
+ Val.has_type v ty ->
+ wt_locset rs ->
+ wt_locset (Locmap.setres res v rs).
+Proof.
+ induction res; simpl; intros.
+- apply wt_setreg; auto. eapply Val.has_subtype; eauto.
+- auto.
+- InvBooleans. eapply IHres2; eauto. destruct v; exact I.
+ eapply IHres1; eauto. destruct v; exact I.
+Qed.
+
Lemma wt_find_label:
forall f lbl c,
wt_function f = true ->
@@ -291,12 +311,8 @@ Proof.
- (* builtin *)
simpl in *; InvBooleans.
econstructor; eauto.
- apply wt_setlist.
- eapply Val.has_subtype_list; eauto. eapply external_call_well_typed'; eauto.
+ eapply wt_setres; eauto. eapply external_call_well_typed; eauto.
apply wt_undef_regs; auto.
-- (* annot *)
- simpl in *; InvBooleans.
- econstructor; eauto.
- (* label *)
simpl in *. econstructor; eauto.
- (* goto *)
@@ -362,10 +378,10 @@ Proof.
intros. inv H. simpl in WTC; InvBooleans. auto.
Qed.
-Lemma wt_state_annot:
- forall s f sp ef args c rs m,
- wt_state (State s f sp (Lannot ef args :: c) rs m) ->
- forallb (loc_valid f) (params_of_annot_args args) = true.
+Lemma wt_state_builtin:
+ forall s f sp ef args res c rs m,
+ wt_state (State s f sp (Lbuiltin ef args res :: c) rs m) ->
+ forallb (loc_valid f) (params_of_builtin_args args) = true.
Proof.
intros. inv H. simpl in WTC; InvBooleans. auto.
Qed.