Skip to content

Commit

Permalink
squash: move in_omonad to Reader_Option_Monad.thy
Browse files Browse the repository at this point in the history
Signed-off-by: Corey Lewis <[email protected]>
  • Loading branch information
corlewis committed Feb 29, 2024
1 parent ce911d2 commit 8610075
Show file tree
Hide file tree
Showing 3 changed files with 2 additions and 4 deletions.
2 changes: 0 additions & 2 deletions lib/Monads/nondet/Nondet_Reader_Option.thy
Original file line number Diff line number Diff line change
Expand Up @@ -130,8 +130,6 @@ lemmas omonad_simps [simp] =
gets_the_throwError gets_the_assert gets_the_Some
gets_the_oapply_comp

lemmas in_omonad = bind_eq_Some_conv in_obind_eq in_opt_map_eq in_opt_pred Let_def


section "Relation between option monad loops and non-deterministic monad loops."

Expand Down
2 changes: 2 additions & 0 deletions lib/Monads/reader_option/Reader_Option_Monad.thy
Original file line number Diff line number Diff line change
Expand Up @@ -482,6 +482,8 @@ lemma obindK_is_opt_map:
"f \<bind> (\<lambda>x. K $ g x) = f |> g"
by (simp add: obind_def opt_map_def)

lemmas in_omonad = bind_eq_Some_conv in_obind_eq in_opt_map_eq in_opt_pred Let_def


section \<open>"While" loops over option monad.\<close>

Expand Down
2 changes: 0 additions & 2 deletions lib/Monads/trace/Trace_Reader_Option.thy
Original file line number Diff line number Diff line change
Expand Up @@ -130,8 +130,6 @@ lemmas omonad_simps [simp] =
gets_the_throwError gets_the_assert gets_the_Some
gets_the_oapply_comp

lemmas in_omonad = bind_eq_Some_conv in_obind_eq in_opt_map_eq in_opt_pred Let_def


section "Relation between option monad loops and trace monad loops."

Expand Down

0 comments on commit 8610075

Please sign in to comment.