Forked from
RT-PROOFS / PROSA - Formally Proven Schedulability Analysis
627 commits behind the upstream repository.
-
Sergey Bozhko authoredSergey Bozhko authored
preemptive.v 628 B
From rt.util Require Import all.
From rt.restructuring.behavior Require Import all.
From rt.restructuring.model.preemption Require Import job.parameters.
(** * Platform for Fully Premptive Model *)
(** In this section, we instantiate [job_preemptable] for the fully
preemptive model. *)
Section FullyPreemptiveModel.
(** Consider any type of jobs. *)
Context {Job : JobType}.
(** In the fully preemptive model any job can be preempted at any time. *)
Global Program Instance fully_preemptive_model : JobPreemptable Job :=
{
job_preemptable (j : Job) (ρ : work) := true
}.
End FullyPreemptiveModel.