Skip to content

Commit

Permalink
lib/monads: add select_wp and alternative_wp to wp set for Nondet monad
Browse files Browse the repository at this point in the history
Signed-off-by: Corey Lewis <[email protected]>
  • Loading branch information
corlewis committed Aug 9, 2023
1 parent aa8b108 commit 0e0e0ca
Showing 1 changed file with 6 additions and 1 deletion.
7 changes: 6 additions & 1 deletion lib/Monads/nondet/Nondet_VCG.thy
Original file line number Diff line number Diff line change
Expand Up @@ -554,7 +554,7 @@ lemma alternativeE_R_wp:
unfolding validE_R_def
by (rule alternativeE_wp)

lemma alternative_R_wp:
lemma alternativeE_E_wp:
"\<lbrakk> \<lbrace>P\<rbrace> f -,\<lbrace>Q\<rbrace>; \<lbrace>P'\<rbrace> g -,\<lbrace>Q\<rbrace> \<rbrakk> \<Longrightarrow> \<lbrace>P and P'\<rbrace> f \<sqinter> g -, \<lbrace>Q\<rbrace>"
unfolding validE_E_def
by (rule alternativeE_wp)
Expand Down Expand Up @@ -1009,6 +1009,11 @@ lemmas [wp] = hoare_vcg_prop
gets_the_wp
gets_map_wp'
liftE_wp
alternative_wp
alternativeE_R_wp
alternativeE_E_wp
alternativeE_wp
select_wp
select_f_wp
state_select_wp
condition_wp
Expand Down

0 comments on commit 0e0e0ca

Please sign in to comment.