Skip to content

Commit

Permalink
squash Trace_Monad_Equations: PR suggestions
Browse files Browse the repository at this point in the history
Signed-off-by: Corey Lewis <[email protected]>
  • Loading branch information
corlewis committed Mar 22, 2024
1 parent 4089a16 commit ee3bc64
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions lib/Monads/trace/Trace_Monad_Equations.thy
Original file line number Diff line number Diff line change
Expand Up @@ -413,11 +413,11 @@ lemma monad_eq_split_tail:

lemma double_gets_drop_regets:
"(do x \<leftarrow> gets f;
xa \<leftarrow> gets f;
m xa x
y \<leftarrow> gets f;
m y x
od) =
(do xa \<leftarrow> gets f;
m xa xa
(do x \<leftarrow> gets f;
m x x
od)"
by (simp add: simpler_gets_def bind_def)

Expand Down

0 comments on commit ee3bc64

Please sign in to comment.