mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-18 08:42:11 +03:00
7 lines
142 B
Idris
7 lines
142 B
Idris
|
module Control.Monad.Trans
|
||
|
|
||
|
public export
|
||
|
interface MonadTrans (t : (Type -> Type) -> Type -> Type) where
|
||
|
lift : Monad m => m a -> t m a
|
||
|
|