Skip to content

Commit

Permalink
lib/monads: rename assert_opt_ovalid to oassert_opt_ovalid and make [wp]
Browse files Browse the repository at this point in the history
Signed-off-by: Michael McInerney <[email protected]>
  • Loading branch information
michaelmcinerney committed Mar 19, 2024
1 parent 688e55b commit 4db52e9
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion lib/Monads/reader_option/Reader_Option_VCG.thy
Original file line number Diff line number Diff line change
Expand Up @@ -129,7 +129,7 @@ lemma owhile_ovalid[wp]:
apply auto
done

lemma assert_opt_ovalid:
lemma oassert_opt_ovalid[wp]:
"\<lblot>\<lambda>s. \<forall>y. x = Some y \<longrightarrow> Q y s\<rblot> oassert_opt x \<lblot>Q\<rblot>"
unfolding oassert_opt_def
by (case_tac x; wpsimp)
Expand Down

0 comments on commit 4db52e9

Please sign in to comment.