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