Library prosa.analysis.facts.priority.edf

We first make some trivial observations about EDF priorities to avoid repeating these steps in subsequent proofs.
Section PriorityFacts.
Consider any type of jobs with arrival times.
  Context `{Job : JobType} `{JobArrival Job}.

First, consider the general case where jobs have arbitrary deadlines.
  Section JobDeadline.

If jobs have arbitrary deadlines ...
    Context `{JobDeadline Job}.

... then hep_job is a statement about these deadlines.
    Fact hep_job_deadline :
       j j',
        hep_job j j' = (job_deadline j job_deadline j').
    Proof. by movej j'; rewrite /hep_job /EDF. Qed.

  End JobDeadline.

Second, consider the case where job (absolute) deadlines are derived from task (relative) deadlines.
  Section TaskDeadline.

If the jobs stem from tasks with relative deadlines ...
    Context {Task : TaskType}.
    Context `{TaskDeadline Task}.
    Context `{JobTask Job Task}.

... then hep_job is a statement about job arrival times and relative deadlines.
    Fact hep_job_task_deadline :
       j j',
        hep_job j j' = (job_arrival j + task_deadline (job_task j)
                         job_arrival j' + task_deadline (job_task j')).
    Proof.
      movej j'.
      by rewrite hep_job_deadline /job_deadline/job_deadline_from_task_deadline.
    Qed.

Furthermore, if we are looking at two jobs of the same task, then hep_job is a statement about their respective arrival times.
    Fact hep_job_arrival_edf :
       j j',
        same_task j j'
        hep_job j j' = (job_arrival j job_arrival j').
    Proof.
      by movej j' /eqP SAME; rewrite hep_job_task_deadline SAME leq_add2r.
    Qed.

EDF respects the sequential-tasks hypothesis.
    Lemma EDF_respects_sequential_tasks :
      policy_respects_sequential_tasks (EDF Job).
    Proof.
      by movej j' /eqP TSK ?; rewrite hep_job_arrival_edf // /same_task TSK.
    Qed.
  End TaskDeadline.

End PriorityFacts.

We add the above lemma into a "Hint Database" basic_rt_facts, so Coq will be able to apply it automatically.
Global Hint Resolve EDF_respects_sequential_tasks : basic_rt_facts.

Require Export prosa.model.task.sequentiality.
Require Export prosa.analysis.facts.priority.inversion.
Require Export prosa.analysis.facts.priority.sequential.
Require Export prosa.analysis.facts.model.sequential.

In this section, we prove that the EDF priority policy implies that tasks are executed sequentially.
Section SequentialEDF.

Consider any type of tasks ...
  Context {Task : TaskType}.
  Context `{TaskCost Task}.
  Context `{TaskDeadline Task}.

... with a bound on the maximum non-preemptive segment length. The bound is needed to ensure that, at any instant, it always exists a subsequent preemption time in which the scheduler can, if needed, switch to another higher-priority job.
Further, consider any type of jobs associated with these tasks.
  Context {Job : JobType}.
  Context `{JobTask Job Task}.
  Context `{Arrival : JobArrival Job}.
  Context `{Cost : JobCost Job}.

Allow for any uniprocessor model.
  Context {PState : ProcessorState Job}.
  Hypothesis H_uniproc : uniprocessor_model PState.

Consider any valid arrival sequence.
Next, consider any schedule of this arrival sequence, ...
  Variable sched : schedule PState.

... allow for any work-bearing notion of job readiness, ...
... and assume that the schedule is valid.
In addition, we assume the existence of a function mapping jobs to their preemption points ...
  Context `{JobPreemptable Job}.

... and assume that it defines a valid preemption model with bounded non-preemptive segments.
Assume an EDF schedule.
To prove sequentiality, we use lemma early_hep_job_is_scheduled. Clearly, under the EDF priority policy, jobs satisfy the conditions described by the lemma (i.e., given two jobs j1 and j2 from the same task, if j1 arrives earlier than j2, then j1 always has a higher priority than job j2, and hence completes before j2); therefore EDF implies sequential tasks.
  Lemma EDF_implies_sequential_tasks :
    sequential_tasks arr_seq sched.
  Proof.
    movej1 j2 t ARR1 ARR2 SAME LT.
    apply: early_hep_job_is_scheduled ⇒ //.
    rewrite always_higher_priority_jlfp !hep_job_arrival_edf //.
    - by rewrite -ltnNge; apply/andP; split ⇒ //.
    - by rewrite same_task_sym.
  Qed.

End SequentialEDF.