- 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
-
- 31 Oct, 2019 1 commit
-
-
Maxime Lesourd authored
- Added unfolding lemmas to basic_facts/ideal - Fixed proofs depending on the previous definition using unfolding lemmas The changes follow the discussion in Paris.
-
- 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 1 commit
-
-
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
-
- 23 Aug, 2019 1 commit
-
-
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
-
- 05 Jun, 2019 2 commits
-
-
Maxime Lesourd authored
-
Maxime Lesourd authored
-
- 16 May, 2019 1 commit
-
-
Björn Brandenburg authored
-