|
Agda.TypeChecking.Monad.Exception |
|
|
Description |
Basically a copy of the ErrorT monad transformer. It's handy to slap
onto TCM and still be a MonadTCM (which isn't possible with ErrorT).
|
|
|
Documentation |
|
newtype ExceptionT err m a | Source |
|
Constructors | ExceptionT | | runExceptionT :: m (Either err a) | |
|
|
|
|
class Error err => MonadException err m | m -> err where | Source |
|
| Methods | throwException :: err -> m a | Source |
| | catchException :: m a -> (err -> m a) -> m a | Source |
|
|
|
|
Produced by Haddock version 2.6.1 |