Skip to content

Commit

Permalink
lib: update for trace refactor
Browse files Browse the repository at this point in the history
Signed-off-by: Corey Lewis <[email protected]>
  • Loading branch information
corlewis committed Aug 15, 2023
1 parent b869736 commit aa3ec99
Show file tree
Hide file tree
Showing 4 changed files with 9 additions and 9 deletions.
3 changes: 2 additions & 1 deletion lib/Crunch_Instances_Trace.thy
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,8 @@
theory Crunch_Instances_Trace
imports
Crunch
Monads.Trace_VCG
Monads.Trace_No_Fail
Monads.Trace_RG
begin

lemmas [crunch_param_rules] = Let_def return_bind returnOk_bindE
Expand Down
7 changes: 4 additions & 3 deletions lib/concurrency/Atomicity_Lib.thy
Original file line number Diff line number Diff line change
Expand Up @@ -5,8 +5,9 @@
*)
theory Atomicity_Lib

imports "Prefix_Refinement"

imports
Prefix_Refinement
Monads.Trace_Det
begin

text \<open>This library introduces a number of proofs about the question of
Expand Down Expand Up @@ -186,7 +187,7 @@ lemma repeat_n_nothing:
lemma repeat_nothing:
"repeat (\<lambda>_. {}) = return ()"
by (simp add: repeat_def bind_def select_def repeat_n_nothing
Sigma_def if_fun_lift UN_If_distrib return_def
Sigma_def if_distribR UN_If_distrib return_def
cong del: image_cong_simp)

lemma detrace_env_steps:
Expand Down
4 changes: 1 addition & 3 deletions lib/concurrency/Prefix_Refinement.thy
Original file line number Diff line number Diff line change
Expand Up @@ -7,8 +7,6 @@ theory Prefix_Refinement

imports
Triv_Refinement
"Monads.Trace_Lemmas"

begin

section \<open>Definition of prefix fragment refinement.\<close>
Expand Down Expand Up @@ -1242,7 +1240,7 @@ lemma prefix_refinement_repeat:
apply simp
apply (rule prefix_refinement_repeat_n, assumption+)
apply (rule validI_weaken_pre, assumption, simp)
apply (wp select_wp)
apply wp
apply wp
apply clarsimp
apply clarsimp
Expand Down
4 changes: 2 additions & 2 deletions lib/concurrency/Triv_Refinement.thy
Original file line number Diff line number Diff line change
Expand Up @@ -6,8 +6,8 @@
theory Triv_Refinement

imports
"Monads.Trace_VCG"
"Monads.Strengthen"
"Monads.Trace_RG"
"Monads.Trace_Strengthen_Setup"

begin

Expand Down

0 comments on commit aa3ec99

Please sign in to comment.