mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-11 02:01:36 +03:00
finished MonadRWS
This commit is contained in:
parent
e906b28cae
commit
d36a234041
@ -2,3 +2,6 @@ module Control.Monad.RWS
|
||||
|
||||
import public Control.Monad.RWS.CPS as Control.Monad.RWS
|
||||
import public Control.Monad.RWS.Interface as Control.Monad.RWS
|
||||
import public Control.Monad.Reader.Interface as Control.Monad.RWS
|
||||
import public Control.Monad.Writer.Interface as Control.Monad.RWS
|
||||
import public Control.Monad.State.Interface as Control.Monad.RWS
|
||||
|
@ -1 +1,13 @@
|
||||
module Control.Monad.RWS.Interface
|
||||
|
||||
import Control.Monad.RWS.CPS
|
||||
import Control.Monad.Reader.Interface
|
||||
import Control.Monad.State.Interface
|
||||
import Control.Monad.Writer.Interface
|
||||
|
||||
public export
|
||||
interface (MonadReader r m, MonadWriter w m, MonadState s m) =>
|
||||
MonadRWS r w s m | m where
|
||||
|
||||
public export
|
||||
(Monoid w, Monad m) => MonadRWS r w s (RWST r w s m) where
|
||||
|
Loading…
Reference in New Issue
Block a user