Idris2Doc : Control.Monad.Partial

Control.Monad.Partial(source)

Definitions

dataPartial : Type->Type
  Delay/partiality monad. Represents partial computations which may not
terminate or cover all inputs. This can be preferable to defining a partial
Idris function as it allows termination to be proven as an external proof.

Totality: total
Visibility: public export
Constructors:
Now : a->Partiala
Later : Inf (Partiala) ->Partiala

Hints:
ApplicativePartial
FunctorPartial
MonadPartial
never : Partiala
  A partial computation which never terminates (aka. undefined/bottom).

Totality: total
Visibility: public export
dataTotal : Partiala->Type
Totality: total
Visibility: public export
Constructors:
TNow : (x : a) ->Total (Nowx)
TLater : Total (Force x) ->Total (Laterx)
runPartial : (0_ : Totalx) ->a
  Extract the value from a partial computation if you have a proof it is
actually total.

Totality: total
Visibility: public export