Skip to content
GitLab
Explore
Sign in
Primary navigation
Search or go to…
Project
P
PROSA - Formally Proven Schedulability Analysis
Manage
Activity
Members
Labels
Plan
Issues
Issue boards
Milestones
Code
Merge requests
Repository
Branches
Commits
Tags
Repository graph
Compare revisions
Build
Pipelines
Jobs
Pipeline schedules
Artifacts
Help
Help
Support
GitLab documentation
Compare GitLab plans
Community forum
Contribute to GitLab
Provide feedback
Terms and privacy
Keyboard shortcuts
?
Snippets
Groups
Projects
Show more breadcrumbs
RT-PROOFS
PROSA - Formally Proven Schedulability Analysis
Commits
9156dbfe
Commit
9156dbfe
authored
1 year ago
by
Kimaya Bedarkar
Committed by
Björn Brandenburg
1 year ago
Browse files
Options
Downloads
Patches
Plain Diff
generalize task-cost inequality lemma
parent
e126e8c3
No related branches found
No related tags found
1 merge request
!327
Generalize one lemma
Pipeline
#97053
passed
1 year ago
Changes
3
Pipelines
1
Hide whitespace changes
Inline
Side-by-side
Showing
3 changed files
analysis/abstract/IBF/task.v
+4
-52
4 additions, 52 deletions
analysis/abstract/IBF/task.v
analysis/facts/model/rbf.v
+118
-1
118 additions, 1 deletion
analysis/facts/model/rbf.v
results/fifo/rta.v
+6
-2
6 additions, 2 deletions
results/fifo/rta.v
with
128 additions
and
55 deletions
analysis/abstract/IBF/task.v
+
4
−
52
View file @
9156dbfe
...
...
@@ -545,56 +545,6 @@ Section TaskIBFtoJobIBF.
End
TaskInterferenceBoundsInterference
.
(** In order to obtain a more convenient bound on the cumulative
interference, we need to abandon the actual workload in favor
of a bound that depends on task parameters only. So, we show
that the actual workload of the task excluding workload of any
job [j] is no greater than the bound on the workload excluding
the cost of job [j]'s task. *)
Lemma
task_rbf_excl_tsk_bounds_task_workload_excl_j
:
task_workload_between
arr_seq
tsk
t1
(
t1
+
A
+
ε
)
-
job_cost
j
<=
task_rbf
(
A
+
ε
)
-
task_cost
tsk
.
Proof
.
move
:
H_j_arrives
H_job_of_tsk
H_busy_interval
=>
ARR
TSK
[[
/
andP
[
JAGET1
JALTT2
]
_]
_]
.
apply
leq_trans
with
(
task_cost
tsk
*
number_of_task_arrivals
arr_seq
tsk
t1
(
t1
+
A
+
ε
)
-
task_cost
tsk
);
last
first
.
{
rewrite
leq_sub2r
//
leq_mul2l
;
apply
/
orP
;
right
.
rewrite
-
addnA
-
{
2
}[(
A
+
1
)](
addKn
t1
)
.
by
apply
H_is_arrival_curve
;
auto
using
leq_addr
.
}
have
Fact6
:
j
\
in
arrivals_between
(
t1
+
A
)
(
t1
+
A
+
ε
)
.
{
apply
arrived_between_implies_in_arrivals
=>
//.
apply
/
andP
;
split
;
rewrite
/
A
subnKC
//.
by
rewrite
addn1
ltnSn
//.
}
have
Fact4
:
j
\
in
arrivals_at
arr_seq
(
t1
+
A
)
.
{
have
CONSISTENT
:
consistent_arrival_times
arr_seq
by
[]
.
by
move
:
ARR
=>
[
t
ARR
];
rewrite
subnKC
//
;
feed
(
CONSISTENT
j
t
);
try
(
subst
t
)
.
}
have
Fact1
:
1
<=
number_of_task_arrivals
arr_seq
tsk
(
t1
+
A
)
(
t1
+
A
+
ε
)
.
{
rewrite
/
number_of_task_arrivals
/
task_arrivals_between
/
arrival_sequence
.
arrivals_between
.
by
rewrite
size_filter
-
has_count
;
apply
/
hasP
;
exists
j
;
last
rewrite
TSK
.
}
rewrite
(
@
num_arrivals_of_task_cat
_
_
_
_
_
(
t1
+
A
));
last
by
apply
/
andP
;
split
;
rewrite
leq_addr
//.
rewrite
mulnDr
.
have
Step1
:
task_workload_between
arr_seq
tsk
t1
(
t1
+
A
+
ε
)
=
task_workload_between
arr_seq
tsk
t1
(
t1
+
A
)
+
task_workload_between
arr_seq
tsk
(
t1
+
A
)
(
t1
+
A
+
ε
)
.
{
by
apply
workload_of_jobs_cat
;
apply
/
andP
;
split
;
rewrite
leq_addr
.
}
rewrite
Step1
;
clear
Step1
.
rewrite
-!
addnBA
;
first
last
.
{
by
rewrite
/
task_workload_between
/
workload
.
task_workload_between
/
task_workload
/
workload_of_jobs
(
big_rem
j
)
//=
TSK
leq_addr
.
}
{
apply
leq_trans
with
(
task_cost
tsk
)
=>
[
//|
]
.
by
rewrite
-
{
1
}[
task_cost
tsk
]
muln1
leq_mul2l
;
apply
/
orP
;
right
.
}
rewrite
leq_add
//
;
first
exact
:
task_workload_le_num_of_arrivals_times_cost
.
rewrite
/
task_workload_between
/
workload
.
task_workload_between
/
task_workload
/
workload_of_jobs
/
arrival_sequence
.
arrivals_between
/
number_of_task_arrivals
/
task_arrivals_between
/
arrival_sequence
.
arrivals_between
.
rewrite
{
1
}
addn1
big_nat1
addn1
big_nat1
.
rewrite
(
big_rem
j
)
//=
TSK
//=
addnC
-
addnBA
//
subnn
addn0
.
rewrite
(
filter_size_rem
j
)
//.
rewrite
mulnDr
mulnC
muln1
-
addnBA
//
subnn
addn0
mulnC
.
apply
sum_majorant_constant
.
move
=>
j'
ARR'
/
eqP
TSK2
.
by
rewrite
-
TSK2
;
apply
H_valid_job_cost
;
exists
(
t1
+
A
);
apply
rem_in
in
ARR'
.
Qed
.
(** We use the lemmas above to obtain the bound on [interference]
in terms of [task_rbf] and [task_interference]. *)
Lemma
cumulative_job_interference_bound
:
...
...
@@ -609,8 +559,10 @@ Section TaskIBFtoJobIBF.
task_workload_between
arr_seq
tsk
t1
(
t1
+
A
+
ε
)
-
job_cost
j
+
cumul_task_interference
arr_seq
sched
j
t1
y
)
.
-
by
apply
cumulative_job_interference_le_task_interference_bound
.
-
rewrite
leq_add2r
.
by
eapply
task_rbf_excl_tsk_bounds_task_workload_excl_j
;
eauto
2
.
-
rewrite
leq_add2r
/
A
.
have
->
:
(
t1
+
(
job_arrival
j
-
t1
)
+
ε
)
=
(
t1
+
(
job_arrival
j
-
t1
+
ε
))
by
lia
.
apply
:
task_rbf_without_job_under_analysis
=>
//=.
by
move
:
IN
=>
/
[
!
job_arrival_in_bounds
]
//
-
[];
lia
.
Qed
.
End
BoundOfCumulativeJobInterference
.
...
...
This diff is collapsed.
Click to expand it.
analysis/facts/model/rbf.v
+
118
−
1
View file @
9156dbfe
...
...
@@ -541,7 +541,6 @@ Section FP_RBF_partitioning.
End
FP_RBF_partitioning
.
(** In this section, we state a few facts for RBFs in the context of a
fixed-priority policy. *)
Section
RBFFOrFP
.
...
...
@@ -611,3 +610,121 @@ Section RBFFOrFP.
Qed
.
End
RBFFOrFP
.
(** We know that the workload of a task in any interval must be
bounded by the task's RBF in that interval. However, in the proofs
of several lemmas, we are required to reason about the workload of
a task in an interval excluding the cost of a particular job
(usually the job under analysis). Such a workload can be tightly
bounded by the task's RBF for the interval excluding the cost of
one task.
Notice, however, that this is not a trivial result since a naive
approach to proving it would fail. Suppose we want to prove that
some quantity [A - B] is upper bounded by some quantity [C -
D]. This usually requires us to prove that [A] is upper bounded by
[C] _and_ [D] is upper bounded by [B]. In our case, this would be
equivalent to proving that the task cost is upper-bounded by the
job cost, which of course is not true.
So, a different approach is needed, which we show in this
section. *)
Section
TaskWorkload
.
(** Consider any type of tasks ... *)
Context
{
Task
:
TaskType
}
.
Context
`{
TaskCost
Task
}
.
(** ... and any type of jobs associated with these tasks. *)
Context
{
Job
:
JobType
}
.
Context
`{
JobTask
Job
Task
}
.
Context
`{
JobArrival
Job
}
.
Context
`{
JobCost
Job
}
.
(** Consider any arrival sequence ... *)
Variable
arr_seq
:
arrival_sequence
Job
.
Hypothesis
H_arrival_times_are_consistent
:
consistent_arrival_times
arr_seq
.
(** ... and assume that WCETs are respected. *)
Hypothesis
H_arrivals_have_valid_job_costs
:
arrivals_have_valid_job_costs
arr_seq
.
(** Let [tsk] be any task ... *)
Variable
tsk
:
Task
.
(** ... characterized by a valid arrival curve. *)
Context
`{
MaxArrivals
Task
}
.
Hypothesis
H_valid_arrival_curve
:
valid_arrival_curve
(
max_arrivals
tsk
)
.
Hypothesis
H_is_arrival_curve
:
respects_max_arrivals
arr_seq
tsk
(
max_arrivals
tsk
)
.
(** Consider any job [j] of [tsk] ... *)
Variable
j
:
Job
.
Hypothesis
H_job_of_task
:
job_of_task
tsk
j
.
(** ... that arrives in the given arrival sequence. *)
Hypothesis
H_j_arrives_in
:
arrives_in
arr_seq
j
.
(** Consider any time instant [t1] and duration [Δ] such that [j]
arrives before [t1 + Δ]. *)
Variables
(
t1
:
instant
)
(
Δ
:
duration
)
.
Hypothesis
H_job_arrival_lt
:
job_arrival
j
<
t1
+
Δ
.
(** As a preparatory step, we restrict our attention to the sub-interval
containing the job's arrival. We know that the job's arrival necessarily
happens in the interval (<<[job_arrival j], t1 + Δ>>). This allows us to
show that the task workload excluding the task cost can be bounded by the
cost of the arrivals in the interval as follows. *)
Lemma
task_rbf_without_job_under_analysis_from_arrival
:
task_workload_between
arr_seq
tsk
(
job_arrival
j
)
(
t1
+
Δ
)
-
job_cost
j
<=
task_cost
tsk
*
number_of_task_arrivals
arr_seq
tsk
(
job_arrival
j
)
(
t1
+
Δ
)
-
task_cost
tsk
.
Proof
.
rewrite
/
task_workload_between
/
workload
.
task_workload_between
/
task_workload
/
workload_of_jobs
/
number_of_task_arrivals
/
task_arrivals_between
.
rewrite
(
big_rem
j
)
//=
addnC
//=
H_job_of_task
addnK
(
filter_size_rem
j
)
//.
rewrite
mulnDr
mulnC
muln1
addnK
mulnC
.
apply
sum_majorant_constant
=>
j'
ARR'
/
eqP
TSK2
.
rewrite
-
TSK2
;
apply
H_arrivals_have_valid_job_costs
.
apply
rem_in
in
ARR'
.
by
eapply
in_arrivals_implies_arrived
=>
//=.
Qed
.
(** To use the above lemma in our final theorem, we require that the arrival
of the job under analysis necessarily happens in the interval we are
considering. *)
Hypothesis
H_j_arrives_after_t
:
t1
<=
job_arrival
j
.
(** Under the above assumption, we can finally establish the desired bound. *)
Lemma
task_rbf_without_job_under_analysis
:
task_workload_between
arr_seq
tsk
t1
(
t1
+
Δ
)
-
job_cost
j
<=
task_request_bound_function
tsk
Δ
-
task_cost
tsk
.
Proof
.
apply
leq_trans
with
(
task_cost
tsk
*
number_of_task_arrivals
arr_seq
tsk
t1
(
t1
+
Δ
)
-
task_cost
tsk
);
last
first
.
-
rewrite
leq_sub2r
//
leq_mul2l
;
apply
/
orP
=>
//=
;
right
.
have
POSE
:
Δ
=
(
t1
+
Δ
-
t1
)
by
lia
.
rewrite
[
in
leqRHS
]
POSE
.
eapply
(
H_is_arrival_curve
t1
(
t1
+
Δ
))
.
by
lia
.
-
rewrite
(
@
num_arrivals_of_task_cat
_
_
_
_
_
(
job_arrival
j
));
last
by
apply
/
andP
;
split
.
rewrite
mulnDr
.
rewrite
/
task_workload_between
/
task_workload
(
workload_of_jobs_cat
_
(
job_arrival
j
)
);
last
by
apply
/
andP
;
split
;
lia
.
rewrite
-!
addnBA
;
first
last
.
+
by
rewrite
/
task_workload_between
/
task_workload
/
workload_of_jobs
(
big_rem
j
)
//=
H_job_of_task
leq_addr
.
+
rewrite
-
{
1
}[
task_cost
tsk
]
muln1
leq_mul2l
;
apply
/
orP
;
right
.
rewrite
/
number_of_task_arrivals
/
task_arrivals_between
.
rewrite
size_filter
-
has_count
;
apply
/
hasP
;
exists
j
;
last
by
rewrite
H_job_of_task
.
apply
(
mem_bigcat
_
Job
_
(
job_arrival
j
)
_);
last
by
apply
job_in_arrivals_at
=>
//=.
rewrite
mem_index_iota
.
by
apply
/
andP
;
split
.
+
have
->
:
job_arrival
j
=
t1
+
(
job_arrival
j
-
t1
)
by
lia
.
have
->
:
t1
+
(
job_arrival
j
-
t1
)
=
job_arrival
j
by
lia
.
rewrite
leq_add
//
;
last
by
apply
task_rbf_without_job_under_analysis_from_arrival
=>
//=.
have
->
:
job_arrival
j
=
t1
+
(
job_arrival
j
-
t1
)
by
lia
.
by
eapply
(
task_workload_le_num_of_arrivals_times_cost
)
=>
//=.
Qed
.
End
TaskWorkload
.
This diff is collapsed.
Click to expand it.
results/fifo/rta.v
+
6
−
2
View file @
9156dbfe
...
...
@@ -313,12 +313,16 @@ Section AbstractRTAforFIFOwithArrivalCurves.
{
by
apply
:
task_rbf_1_ge_task_cost
;
exact
:
non_pathological_max_arrivals
.
}
{
by
apply
task_rbf_monotone
;
[
apply
H_valid_arrival_curve
|
lia
]
.
}
-
eapply
leq_trans
;
last
by
erewrite
leq_add2l
;
eapply
task_rbf_excl_tsk_bounds_task_workload_excl_j
;
eauto
1
.
last
by
(
erewrite
leq_add2l
;
eapply
task_rbf_without_job_under_analysis
with
(
t1
:=
t1
)
=>
//
;
lia
)
.
rewrite
addnBA
.
+
rewrite
leq_sub2r
//
;
eapply
leq_trans
.
*
apply
sum_over_partitions_le
=>
j'
inJOBS
=>
_
.
by
apply
H_all_jobs_from_taskset
,
(
in_arrivals_implies_arrived
_
_
_
_
inJOBS
)
.
*
rewrite
(
big_rem
tsk
)
//=
addnC
leq_add
//
;
last
by
rewrite
subnKC
.
*
rewrite
(
big_rem
tsk
)
//=
addnC
leq_add
//
;
last
by
rewrite
addnBAC
//=
subnKC
//
addn1
;
apply
leqW
.
rewrite
big_seq_cond
[
in
X
in
_
<=
X
]
big_seq_cond
big_mkcond
[
in
X
in
_
<=
X
]
big_mkcond
//=.
apply
leq_sum
=>
tsk'
_;
rewrite
andbC
//=.
destruct
(
tsk'
\
in
rem
(
T
:=
Task
)
tsk
ts
)
eqn
:
IN
;
last
by
[]
.
...
...
This diff is collapsed.
Click to expand it.
Preview
0%
Loading
Try again
or
attach a new file
.
Cancel
You are about to add
0
people
to the discussion. Proceed with caution.
Finish editing this message first!
Save comment
Cancel
Please
register
or
sign in
to comment