Skip to content

Commit

Permalink
lib: consistent Trace filename prefix
Browse files Browse the repository at this point in the history
Signed-off-by: Corey Lewis <[email protected]>
  • Loading branch information
corlewis committed Jul 19, 2023
1 parent a8e7256 commit dea1bb8
Show file tree
Hide file tree
Showing 9 changed files with 13 additions and 13 deletions.
2 changes: 1 addition & 1 deletion lib/Crunch_Instances_Trace.thy
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@
theory Crunch_Instances_Trace
imports
Crunch
Monads.TraceMonadVCG
Monads.Trace_VCG
begin

lemmas [crunch_param_rules] = Let_def return_bind returnOk_bindE
Expand Down
2 changes: 1 addition & 1 deletion lib/Monads/Monad_Lib.thy
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
*)

(* This theory collects the minimum constant definitions and lemmas for the monad definition
theories (Nondet_Monad, TraceMonad etc). Only things that are necessary for these and needed
theories (Nondet_Monad, Trace_Monad etc). Only things that are necessary for these and needed
by more than one of them should go in here. *)

theory Monad_Lib
Expand Down
2 changes: 1 addition & 1 deletion lib/Monads/README.md
Original file line number Diff line number Diff line change
Expand Up @@ -35,5 +35,5 @@ in weakest-precondition style.
[l4v]: https://github.com/seL4/l4v/
[nondet]: ./nondet/Nondet_Monad.thy
[option]: ./reader_option/Reader_Option_Monad.thy
[trace]: ./trace/TraceMonad.thy
[trace]: ./trace/Trace_Monad.thy
[AutoCorres]: ../../tools/autocorres/
6 changes: 3 additions & 3 deletions lib/Monads/ROOT
Original file line number Diff line number Diff line change
Expand Up @@ -22,17 +22,17 @@ session Monads (lib) = HOL +

theories
Nondet_WhileLoopRules
TraceMonad
Trace_Monad
Reader_Option_ND
Reader_Option_VCG
Strengthen_Demo
TraceMonadLemmas
Trace_Lemmas
Datatype_Schematic
Nondet_WhileLoopRulesCompleteness
Strengthen
Nondet_Strengthen_Setup
Reader_Option_Monad
TraceMonadVCG
Trace_VCG
Nondet_In_Monad
Nondet_VCG
Nondet_Sat
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,8 @@
*
* SPDX-License-Identifier: BSD-2-Clause
*)
theory TraceMonadLemmas
imports TraceMonadVCG
theory Trace_Lemmas
imports Trace_VCG
begin

lemma mapM_Cons:
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@
*
* SPDX-License-Identifier: BSD-2-Clause
*)
theory TraceMonad
theory Trace_Monad
imports
Monad_Lib
Strengthen
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,9 @@
*
* SPDX-License-Identifier: BSD-2-Clause
*)
theory TraceMonadVCG
theory Trace_VCG
imports
TraceMonad
Trace_Monad
Fun_Pred_Syntax
WPSimp
begin
Expand Down
2 changes: 1 addition & 1 deletion lib/concurrency/Prefix_Refinement.thy
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@ theory Prefix_Refinement

imports
Triv_Refinement
"Monads.TraceMonadLemmas"
"Monads.Trace_Lemmas"

begin

Expand Down
2 changes: 1 addition & 1 deletion lib/concurrency/Triv_Refinement.thy
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@
theory Triv_Refinement

imports
"Monads.TraceMonadVCG"
"Monads.Trace_VCG"
"Monads.Strengthen"

begin
Expand Down

0 comments on commit dea1bb8

Please sign in to comment.