Skip to content

Commit

Permalink
fix indent squash into mapM rules
Browse files Browse the repository at this point in the history
Signed-off-by: Michael McInerney <[email protected]>
  • Loading branch information
michaelmcinerney committed Dec 19, 2024
1 parent aa8cfff commit 96a3752
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion lib/Monad_Lists.thy
Original file line number Diff line number Diff line change
Expand Up @@ -516,7 +516,7 @@ lemma mapM_gets_the_wp:
"\<lbrace>\<lambda>s. \<forall>vs. map (\<lambda>t. f t s) ts = map Some vs \<longrightarrow> P vs s\<rbrace>
mapM (gets_the \<circ> f) ts
\<lbrace>P\<rbrace>"
unfolding comp_def
unfolding comp_def
proof (induct ts arbitrary: P)
case Nil thus ?case by (wpsimp simp: mapM_Nil)
next
Expand Down

0 comments on commit 96a3752

Please sign in to comment.