Library prosa.analysis.facts.model.sbf.average

SBF for Average Resource Model in Valid

In this file, we prove that the SBF defined in the file prosa.analysis.definitions.sbf.average is valid under the average resource model.
Consider any type of tasks ...
  Context {Task : TaskType}.

... and any type of jobs associated with these tasks.
  Context {Job : JobType}.
  Context `{JobTask Job Task}.
  Context `{JobArrival Job}.
  Context `{JobCost Job}.

Consider any kind of processor state.
  Context {PState : ProcessorState Job}.

Consider a JLFP policy, ...
  Context `{JLFP_policy Job}.

... any arrival sequence, ...
  Variable arr_seq : arrival_sequence Job.

... and any schedule.
  Variable sched : schedule PState.

Assume the average resource model with a resource period Π, resource allocation time Θ, and supply delay ν.
We show that sbf is monotone.
  Lemma arm_sbf_monotone : sbf_is_monotone (arm_sbf Π Θ ν).
  Proof.
    moveδ1 δ2 LE; rewrite /arm_sbf.
    interval_to_duration δ1 δ2 Δ.
    apply leq_div2r, leq_mul; lia.
  Qed.

The introduced SBF is also a unit-supply SBF.
  Lemma arm_sbf_unit : unit_supply_bound_function (arm_sbf Π Θ ν).
  Proof.
    move: H_average_resource_model ⇒ [LEΠ _].
    moveδ; rewrite /arm_sbf.
    have [Z|POS] := posnP Π; first by subst; lia.
    have [LEν|LEν] := leqP δ ν.
    { move: (LEν); rewrite -subn_eq0 ⇒ /eqP →.
      have [EQ|EQ]: (δ.+1 - ν = 0) (δ.+1 - ν = 1) by lia.
      { by rewrite EQ. }
      { rewrite EQ //=; clear EQ.
        rewrite mul1n mul0n. rewrite div0n.
        rewrite -(@leq_pmul2r Π) // mul1n.
        by apply: leq_trans; first by apply leq_divM.
      }
    }
    { rewrite -addn1 -addnBAC ?addn1; last by lia.
      by rewrite -addn1 mulnDl mul1n -addn1 -divnDMl //; apply leq_div2r; lia.
    }
  Qed.

Finally, we show that the defined sbf is a valid SBF.
  Lemma arm_sbf_valid :
    valid_supply_bound_function arr_seq sched (arm_sbf Π Θ ν).
  Proof.
    have FS: a, 0 - a = 0 by lia.
    split; first by rewrite /arm_sbf !FS mul0n div0n.
    movej t1 t2 ARR _ t /andP [LE1 LE2].
    move: H_average_resource_model ⇒ [LE SUP].
    interval_to_duration t1 t Δ.
    rewrite /arm_sbf -(leqRW (SUP _ _)) /arm_sbf.
    rewrite addKn.
    lia.
  Qed.

End AverageResourceModelValidSBF.