Computation of resource bounds for Linear code.
Require Import Coqlib.
Require Import Maps.
Require Import AST.
Require Import Op.
Require Import Locations.
Require Import Linear.
Require Import Lineartyping.
Require Import Conventions.
Resource bounds for a function
The bounds record capture how many local and outgoing stack slots
and callee-save registers are used by a function.
We demand that all bounds are positive or null.
These properties are used later to reason about the layout of
the activation record.
Record bounds :
Type :=
mkbounds {
bound_int_local:
Z;
bound_float_local:
Z;
bound_int_callee_save:
Z;
bound_float_callee_save:
Z;
bound_outgoing:
Z;
bound_stack_data:
Z;
bound_int_local_pos:
bound_int_local >= 0;
bound_float_local_pos:
bound_float_local >= 0;
bound_int_callee_save_pos:
bound_int_callee_save >= 0;
bound_float_callee_save_pos:
bound_float_callee_save >= 0;
bound_outgoing_pos:
bound_outgoing >= 0;
bound_stack_data_pos:
bound_stack_data >= 0
}.
The following predicates define the correctness of a set of bounds
for the code of a function.
Section BELOW.
Variable funct:
function.
Variable b:
bounds.
Definition mreg_within_bounds (
r:
mreg) :=
match mreg_type r with
|
Tint =>
index_int_callee_save r <
bound_int_callee_save b
|
Tfloat =>
index_float_callee_save r <
bound_float_callee_save b
end.
Definition slot_within_bounds (
s:
slot) :=
match s with
|
Local ofs Tint => 0 <=
ofs <
bound_int_local b
|
Local ofs Tfloat => 0 <=
ofs <
bound_float_local b
|
Outgoing ofs ty => 0 <=
ofs /\
ofs +
typesize ty <=
bound_outgoing b
|
Incoming ofs ty =>
In (
S s) (
loc_parameters funct.(
fn_sig))
end.
Definition instr_within_bounds (
i:
instruction) :=
match i with
|
Lgetstack s r =>
slot_within_bounds s /\
mreg_within_bounds r
|
Lsetstack r s =>
slot_within_bounds s
|
Lop op args res =>
mreg_within_bounds res
|
Lload chunk addr args dst =>
mreg_within_bounds dst
|
Lcall sig ros =>
size_arguments sig <=
bound_outgoing b
|
Lbuiltin ef args res =>
mreg_within_bounds res
|
Lannot ef args =>
forall s,
In (
S s)
args ->
slot_within_bounds s
|
_ =>
True
end.
End BELOW.
Definition function_within_bounds (
f:
function) (
b:
bounds) :
Prop :=
forall instr,
In instr f.(
fn_code) ->
instr_within_bounds f b instr.
Inference of resource bounds for a function
The resource bounds for a function are computed by a linear scan
of its instructions.
Section BOUNDS.
Variable f:
function.
In the proof of the Stacking pass, we only need to bound the
registers written by an instruction. Therefore, this function
returns these registers, ignoring registers used only as
arguments.
Definition regs_of_instr (
i:
instruction) :
list mreg :=
match i with
|
Lgetstack s r =>
r ::
nil
|
Lsetstack r s =>
r ::
nil
|
Lop op args res =>
res ::
nil
|
Lload chunk addr args dst =>
dst ::
nil
|
Lstore chunk addr args src =>
nil
|
Lcall sig ros =>
nil
|
Ltailcall sig ros =>
nil
|
Lbuiltin ef args res =>
res ::
nil
|
Lannot ef args =>
nil
|
Llabel lbl =>
nil
|
Lgoto lbl =>
nil
|
Lcond cond args lbl =>
nil
|
Ljumptable arg tbl =>
nil
|
Lreturn =>
nil
end.
Fixpoint slots_of_locs (
l:
list loc) :
list slot :=
match l with
|
nil =>
nil
|
S s ::
l' =>
s ::
slots_of_locs l'
|
R r ::
l' =>
slots_of_locs l'
end.
Definition slots_of_instr (
i:
instruction) :
list slot :=
match i with
|
Lgetstack s r =>
s ::
nil
|
Lsetstack r s =>
s ::
nil
|
Lannot ef args =>
slots_of_locs args
|
_ =>
nil
end.
Definition max_over_list (
A:
Type) (
valu:
A ->
Z) (
l:
list A) :
Z :=
List.fold_left (
fun m l =>
Zmax m (
valu l))
l 0.
Definition max_over_instrs (
valu:
instruction ->
Z) :
Z :=
max_over_list instruction valu f.(
fn_code).
Definition max_over_regs_of_instr (
valu:
mreg ->
Z) (
i:
instruction) :
Z :=
max_over_list mreg valu (
regs_of_instr i).
Definition max_over_slots_of_instr (
valu:
slot ->
Z) (
i:
instruction) :
Z :=
max_over_list slot valu (
slots_of_instr i).
Definition max_over_regs_of_funct (
valu:
mreg ->
Z) :
Z :=
max_over_instrs (
max_over_regs_of_instr valu).
Definition max_over_slots_of_funct (
valu:
slot ->
Z) :
Z :=
max_over_instrs (
max_over_slots_of_instr valu).
Definition int_callee_save (
r:
mreg) := 1 +
index_int_callee_save r.
Definition float_callee_save (
r:
mreg) := 1 +
index_float_callee_save r.
Definition int_local (
s:
slot) :=
match s with Local ofs Tint => 1 +
ofs |
_ => 0
end.
Definition float_local (
s:
slot) :=
match s with Local ofs Tfloat => 1 +
ofs |
_ => 0
end.
Definition outgoing_slot (
s:
slot) :=
match s with Outgoing ofs ty =>
ofs +
typesize ty |
_ => 0
end.
Definition outgoing_space (
i:
instruction) :=
match i with Lcall sig _ =>
size_arguments sig |
_ => 0
end.
Lemma max_over_list_pos:
forall (
A:
Type) (
valu:
A ->
Z) (
l:
list A),
max_over_list A valu l >= 0.
Proof.
intros until valu.
unfold max_over_list.
assert (
forall l z,
fold_left (
fun x y =>
Zmax x (
valu y))
l z >=
z).
induction l;
simpl;
intros.
omega.
apply Zge_trans with (
Zmax z (
valu a)).
auto.
apply Zle_ge.
apply Zmax1.
auto.
Qed.
Lemma max_over_slots_of_funct_pos:
forall (
valu:
slot ->
Z),
max_over_slots_of_funct valu >= 0.
Proof.
intros.
unfold max_over_slots_of_funct.
unfold max_over_instrs.
apply max_over_list_pos.
Qed.
Lemma max_over_regs_of_funct_pos:
forall (
valu:
mreg ->
Z),
max_over_regs_of_funct valu >= 0.
Proof.
intros.
unfold max_over_regs_of_funct.
unfold max_over_instrs.
apply max_over_list_pos.
Qed.
Program Definition function_bounds :=
mkbounds
(
max_over_slots_of_funct int_local)
(
max_over_slots_of_funct float_local)
(
max_over_regs_of_funct int_callee_save)
(
max_over_regs_of_funct float_callee_save)
(
Zmax (
max_over_instrs outgoing_space)
(
max_over_slots_of_funct outgoing_slot))
(
Zmax f.(
fn_stacksize) 0)
(
max_over_slots_of_funct_pos int_local)
(
max_over_slots_of_funct_pos float_local)
(
max_over_regs_of_funct_pos int_callee_save)
(
max_over_regs_of_funct_pos float_callee_save)
_ _.
Next Obligation.
Next Obligation.
We now show the correctness of the inferred bounds.
Lemma max_over_list_bound:
forall (
A:
Type) (
valu:
A ->
Z) (
l:
list A) (
x:
A),
In x l ->
valu x <=
max_over_list A valu l.
Proof.
intros until x.
unfold max_over_list.
assert (
forall c z,
let f :=
fold_left (
fun x y =>
Zmax x (
valu y))
c z in
z <=
f /\ (
In x c ->
valu x <=
f)).
induction c;
simpl;
intros.
split.
omega.
tauto.
elim (
IHc (
Zmax z (
valu a)));
intros.
split.
apply Zle_trans with (
Zmax z (
valu a)).
apply Zmax1.
auto.
intro H1;
elim H1;
intro.
subst a.
apply Zle_trans with (
Zmax z (
valu x)).
apply Zmax2.
auto.
auto.
intro.
elim (
H l 0);
intros.
auto.
Qed.
Lemma max_over_instrs_bound:
forall (
valu:
instruction ->
Z)
i,
In i f.(
fn_code) ->
valu i <=
max_over_instrs valu.
Proof.
Lemma max_over_regs_of_funct_bound:
forall (
valu:
mreg ->
Z)
i r,
In i f.(
fn_code) ->
In r (
regs_of_instr i) ->
valu r <=
max_over_regs_of_funct valu.
Proof.
Lemma max_over_slots_of_funct_bound:
forall (
valu:
slot ->
Z)
i s,
In i f.(
fn_code) ->
In s (
slots_of_instr i) ->
valu s <=
max_over_slots_of_funct valu.
Proof.
Lemma int_callee_save_bound:
forall i r,
In i f.(
fn_code) ->
In r (
regs_of_instr i) ->
index_int_callee_save r <
bound_int_callee_save function_bounds.
Proof.
Lemma float_callee_save_bound:
forall i r,
In i f.(
fn_code) ->
In r (
regs_of_instr i) ->
index_float_callee_save r <
bound_float_callee_save function_bounds.
Proof.
Lemma int_local_slot_bound:
forall i ofs,
In i f.(
fn_code) ->
In (
Local ofs Tint) (
slots_of_instr i) ->
ofs <
bound_int_local function_bounds.
Proof.
Lemma float_local_slot_bound:
forall i ofs,
In i f.(
fn_code) ->
In (
Local ofs Tfloat) (
slots_of_instr i) ->
ofs <
bound_float_local function_bounds.
Proof.
Lemma outgoing_slot_bound:
forall i ofs ty,
In i f.(
fn_code) ->
In (
Outgoing ofs ty) (
slots_of_instr i) ->
ofs +
typesize ty <=
bound_outgoing function_bounds.
Proof.
Lemma size_arguments_bound:
forall sig ros,
In (
Lcall sig ros)
f.(
fn_code) ->
size_arguments sig <=
bound_outgoing function_bounds.
Proof.
Consequently, all machine registers or stack slots mentioned by one
of the instructions of function f are within bounds.
Lemma mreg_is_within_bounds:
forall i,
In i f.(
fn_code) ->
forall r,
In r (
regs_of_instr i) ->
mreg_within_bounds function_bounds r.
Proof.
Lemma slot_is_within_bounds:
forall i,
In i f.(
fn_code) ->
forall s,
In s (
slots_of_instr i) ->
Lineartyping.slot_valid f s ->
slot_within_bounds f function_bounds s.
Proof.
Lemma slots_of_locs_charact:
forall s l,
In s (
slots_of_locs l) <->
In (
S s)
l.
Proof.
induction l; simpl; intros.
tauto.
destruct a; simpl; intuition congruence.
Qed.
It follows that every instruction in the function is within bounds,
in the sense of the instr_within_bounds predicate.
Lemma instr_is_within_bounds:
forall i,
In i f.(
fn_code) ->
Lineartyping.wt_instr f i ->
instr_within_bounds f function_bounds i.
Proof.
Lemma function_is_within_bounds:
Lineartyping.wt_code f f.(
fn_code) ->
function_within_bounds f function_bounds.
Proof.
End BOUNDS.