Documentation
Lean
.
Elab
.
Print
Search
return to top
source
Imports
Lean.Elab.Command
Lean.Meta.Eqns
Lean.Util.CollectAxioms
Imported by
Lean
.
Elab
.
Command
.
elabPrint
Lean
.
Elab
.
Command
.
elabPrintAxioms
Lean
.
Elab
.
Command
.
elabPrintEqns
source
def
Lean
.
Elab
.
Command
.
elabPrint
:
CommandElab
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Command
.
elabPrintAxioms
:
CommandElab
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Command
.
elabPrintEqns
:
CommandElab
Equations
Lean.Elab.Command.elabPrintEqns
stx
=
do let
cs
←
Lean.Elab.Command.liftCoreM
(
Lean.Elab.realizeGlobalConstWithInfos
stx
[
2
]
)
cs
.
forM
Lean.Elab.Command.printEqnsOf✝
Instances For