minor MonadWriter cleanup

This commit is contained in:
stefan-hoeck 2021-01-20 05:27:56 +01:00
parent 313f52a88a
commit b6e5ba0830

View File

@ -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 ()