mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-11 02:01:36 +03:00
minor MonadWriter cleanup
This commit is contained in:
parent
313f52a88a
commit
b6e5ba0830
@ -22,8 +22,7 @@ public export
|
||||
interface (Monoid w, Monad m) => MonadWriter w m | m where
|
||||
||| `writer (a,w)` embeds a simple writer action.
|
||||
writer : (a,w) -> m a
|
||||
writer (a, w) = do tell w
|
||||
pure a
|
||||
writer (a, w) = tell w $> a
|
||||
|
||||
||| `tell w` is an action that produces the output `w`.
|
||||
tell : w -> m ()
|
||||
|
Loading…
Reference in New Issue
Block a user