Library prosa.analysis.facts.edf_definitions

Equivalence of EDF Definitions

Recall that we have defined "EDF schedules" in two ways.
The generic way to define an EDF schedule is by using the EDF priority policy defined in model.priority.edf and the general notion of priority-compliant schedules defined in model.schedule.priority_driven.
Another, more straight-forward way to define an EDF schedule is the standalone definition given in model.schedule.edf, which is less general but simpler and used in the EDF optimality proof.
In this file, we show that both definitions are equivalent assuming:
(1) ideal uniprocessor schedules, ...
Require Import prosa.model.processor.ideal.

... (2) the classic Liu & Layland model of readiness without jitter and without self-suspensions, where pending jobs are always ready, and ...
Require Import prosa.model.readiness.basic.

... (3) that jobs are fully preemptive.
For any given type of jobs, each characterized by an arrival time, an execution cost, and an absolute deadline, ...
  Context {Job : JobType} `{JobCost Job} `{JobDeadline Job} `{JobArrival Job}.

...consider a given valid job arrival sequence ...
...and a corresponding schedule.
Suppose jobs don't execute after their completion, ...
...all jobs come from the arrival sequence arr_seq, ...
...and jobs from arr_seq don't miss their deadlines.
We first show that a schedule that satisfies the standalone EDF_schedule predicate is also compliant with the generic notion of EDF policy defined in Prosa, namely the respects_policy_at_preemption_point predicate.
  Lemma EDF_schedule_implies_respects_policy_at_preemption_point :
    EDF_schedule sched
    respects_policy_at_preemption_point arr_seq sched.
  Proof.
    moveEDF j' j t ARR PREEMPTION BL SCHED.
    have suff: t' : nat, t t' < job_deadline j' scheduled_at sched j' t'.
    { move⇒ [t' [/andP [LE _] SCHED']].
      apply: (EDF t); [done | exact LE | exact SCHED' |].
      by apply: (backlogged_implies_arrived sched j' t). }
    apply; apply: incomplete_implies_scheduled_later;
      first by apply: H_no_deadline_misses ⇒ //.
    by apply: (backlogged_implies_incomplete sched j' t).
  Qed.

Conversely, the reverse direction also holds: a schedule that satisfies the respects_policy_at_preemption_point predicate is also an EDF schedule in the sense of EDF_schedule.
  Lemma respects_policy_at_preemption_point_implies_EDF_schedule :
    respects_policy_at_preemption_point arr_seq sched
    EDF_schedule sched.
  Proof.
    moveH_priority_driven t j_hp SCHED t' j LEQ SCHED' EARLIER_ARR.
    case (boolP (j == j_hp)); first by move /eqPEQ; subst.
    move /neqPNEQ.
    exploit (H_priority_driven j j_hp t) ⇒ //.
    { by apply (H_from_arr_seq _ _ SCHED'). }
    { by rewrite /preemption_time; destruct (sched t). }
    { apply /andP; split ⇒ //.
      - apply /andP; split ⇒ //.
        apply (incompletion_monotonic _ j _ _ LEQ).
        apply scheduled_implies_not_completed ⇒ //.
        by apply ideal_proc_model_ensures_ideal_progress.
      - apply /negP; moveSCHED''.
        by exploit (ideal_proc_model_is_a_uniprocessor_model j j_hp sched t). }
  Qed.

From the two preceding lemmas, it follows immediately that the two EDF definitions are indeed equivalent, which we note with the following corollary.