def
Lean.Elab.elabSetOption
{m : Type → Type}
[Monad m]
[MonadOptions m]
[MonadExceptOf Exception m]
[MonadRef m]
[AddErrorMessageContext m]
[MonadLiftT (EIO Exception) m]
[MonadInfoTree m]
(id val : Syntax)
:
m Options
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.elabSetOption.setOption
{m : Type → Type}
[Monad m]
[MonadOptions m]
[MonadExceptOf Exception m]
[MonadRef m]
[AddErrorMessageContext m]
(optionName : Name)
(decl : OptionDecl)
(val : DataValue)
:
m Options
Equations
- One or more equations did not get rendered due to their size.