- 03 Dec, 2019 1 commit
-
-
Sergey Bozhko authored
-
- 19 Nov, 2019 2 commits
-
-
Björn Brandenburg authored
This fixes all warnings about ambiguous module names and resolves #49. It also highlights that we still need to cut down on superfluous Require Import commands in recently ported files.
-
Sergey Bozhko authored
-
- 15 Nov, 2019 2 commits
-
-
Björn Brandenburg authored
-
Björn Brandenburg authored
-
- 16 Oct, 2019 1 commit
-
-
Björn Brandenburg authored
This avoids the need to use @-notation when establishing platform properties (e.g., in facts about ideal schedules). Thanks to Maxime for the suggestion.
-
- 15 Oct, 2019 3 commits
-
-
Björn Brandenburg authored
-
Maxime Lesourd authored
-
Björn Brandenburg authored
-
- 30 Aug, 2019 2 commits
-
-
Björn Brandenburg authored
Rationale: reserve the behavior folder for trace-based semantics. These lemmas really constitute an analysis of the basic consequences arising from the chosen semantics and hence logically belong to the "analysis" part of Prosa.
-
Björn Brandenburg authored
-
- 13 Aug, 2019 1 commit
-
-
Björn Brandenburg authored
To allow reasoning about an entire class of types of schedules / processor modules, it's useful to have named definitions for various invariants that processor models ensure. Let's collect these centrally where we introduce processor models and schedules.
-
- 26 Jun, 2019 1 commit
-
-
Maxime Lesourd authored
simplify structure of behavior, move arrival_sequence and schedule to toplevel, move task and sequential to model
-
- 25 Jun, 2019 1 commit
-
-
Björn Brandenburg authored
- Consistently use JobType rather than eqType directly. - Fix the comments style.
-
- 05 Jun, 2019 1 commit
-
-
Maxime Lesourd authored
-
- 16 May, 2019 4 commits
-
-
Björn Brandenburg authored
...and introduce a bunch of helper lemmas to get there.
-
Björn Brandenburg authored
Let's not clutter up the spec with facts files all over the place. Instead, let's collect the facts files in a separate folder / hierarchy.
-
Björn Brandenburg authored
- port completed_implies_scheduled_before - port lemmas on service prior to arrival - port scheduled_implies_pending and greatly simplify the proof while at it - port and simplify job_pending_at_arrival - port cumulative_service_implies_scheduled and simplify proof of positive_service_implies_scheduled_before - port service_is_a_step_function
-
Björn Brandenburg authored
-
- 13 May, 2019 1 commit
-
-
Björn Brandenburg authored
...from model/schedule/uni/schedule.v. To simplify some of the rather long proofs in the original file, the patch introduces a bunch of small and simple rewriting and helper lemmas that we previously lacked, but that we *should* have to avoid having to reason at the level of sslreflect "big" operators in every lemma.
-