clarify toMaybeT docstring

This commit is contained in:
Joel Berkeley 2024-05-05 15:57:27 +01:00 committed by G. Allais
parent c0ac024114
commit 40d4cd898b

View File

@ -68,7 +68,9 @@ public export
fromMaybeT : Monad m => m a -> MaybeT m a -> m a
fromMaybeT v x = runMaybeT x >>= maybe v pure
||| Return a value if a condition is met, or else no value.
||| Return a value if a condition is met, or else no value. The condition
||| only affects whether the `Maybe` produces a value; the effect is run
||| either way.
|||
||| This is a version of `toMaybe` lifted to work with `MaybeT`.
public export