Idris2/libs/base/Control/Monad/Trans.idr
Jeremy 394613432f
Add documentation for Control.Monad.* (#2365)
Co-authored-by: Zoe Stafford <36511192+Z-snails@users.noreply.github.com>
2022-03-25 10:14:25 +00:00

11 lines
304 B
Idris

module Control.Monad.Trans
%default total
||| A monad transformer is a type that can wrap an inner monad, extending it
||| with additional abilities.
public export
interface MonadTrans t where
||| Lift a computation from the inner monad to the transformed monad.
lift : Monad m => m a -> t m a