Documentation
Lake
.
DSL
.
Meta
Search
return to top
source
Imports
Lean.ToExpr
Lake.DSL.Syntax
Lake.Util.FilePath
Lean.Elab.ElabRules
Lean.Elab.Eval
Imported by
Lake
.
DSL
.
toExprIO
Syntax for elaboration time control flow.
source
def
Lake
.
DSL
.
toExprIO
{
α
:
Type
}
[
Lean.ToExpr
α
]
(
x
:
IO
α
)
:
IO
Lean.Expr
Equations
Lake.DSL.toExprIO
x
=
Lean.toExpr
<$>
x
Instances For