mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-22 19:21:39 +03:00
394613432f
Co-authored-by: Zoe Stafford <36511192+Z-snails@users.noreply.github.com>
11 lines
304 B
Idris
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
|