Documentation
Lean
.
Compiler
.
IR
Search
Google site search
return to top
source
Imports
Lean.Compiler.IR.Basic
Lean.Compiler.IR.Borrow
Lean.Compiler.IR.Boxing
Lean.Compiler.IR.Checker
Lean.Compiler.IR.CompilerM
Lean.Compiler.IR.CtorLayout
Lean.Compiler.IR.ElimDeadBranches
Lean.Compiler.IR.ElimDeadVars
Lean.Compiler.IR.EmitC
Lean.Compiler.IR.ExpandResetReuse
Lean.Compiler.IR.Format
Lean.Compiler.IR.NormIds
Lean.Compiler.IR.PushProj
Lean.Compiler.IR.RC
Lean.Compiler.IR.ResetReuse
Lean.Compiler.IR.SimpCase
Lean.Compiler.IR.Sorry
Lean.Compiler.IR.UnboxResult
Imported by
Lean
.
IR
.
compiler
.
reuse
Lean
.
IR
.
compile
Lean
.
IR
.
addBoxedVersionAux
Lean
.
IR
.
addBoxedVersion
source
opaque
Lean
.
IR
.
compiler
.
reuse
:
Lean.Option
Bool
source
@[export lean_ir_compile]
def
Lean
.
IR
.
compile
(env :
Lean.Environment
)
(opts :
Lean.Options
)
(decls :
Array
Lean.IR.Decl
)
:
Lean.IR.Log
×
Except
String
Lean.Environment
Instances For
source
def
Lean
.
IR
.
addBoxedVersionAux
(decl :
Lean.IR.Decl
)
:
Lean.IR.CompilerM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For
source
@[export lean_ir_add_boxed_version]
def
Lean
.
IR
.
addBoxedVersion
(env :
Lean.Environment
)
(decl :
Lean.IR.Decl
)
:
Except
String
Lean.Environment
Equations
One or more equations did not get rendered due to their size.
Instances For