Documentation
Lean
.
Meta
.
PPGoal
Search
return to top
source
Imports
Lean.Meta.InferType
Imported by
Lean
.
Meta
.
pp
.
auxDecls
Lean
.
Meta
.
pp
.
implementationDetailHyps
Lean
.
Meta
.
pp
.
inaccessibleNames
Lean
.
Meta
.
pp
.
showLetValues
Lean
.
Meta
.
getGoalPrefix
Lean
.
Meta
.
ppGoal
Lean
.
Meta
.
ppGoal
.
pushPending
Lean
.
Meta
.
ppGoal
.
ppVars
source
opaque
Lean
.
Meta
.
pp
.
auxDecls
:
Lean.Option
Bool
source
opaque
Lean
.
Meta
.
pp
.
implementationDetailHyps
:
Lean.Option
Bool
source
opaque
Lean
.
Meta
.
pp
.
inaccessibleNames
:
Lean.Option
Bool
source
opaque
Lean
.
Meta
.
pp
.
showLetValues
:
Lean.Option
Bool
source
def
Lean
.
Meta
.
getGoalPrefix
(mvarDecl :
MetavarDecl
)
:
String
Equations
Lean.Meta.getGoalPrefix
mvarDecl
=
if
(
Lean.isLHSGoal?
mvarDecl
.type
)
.isSome
=
true
then
"| "
else
"⊢ "
Instances For
source
def
Lean
.
Meta
.
ppGoal
(mvarId :
MVarId
)
:
MetaM
Format
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
ppGoal
.
pushPending
(indent :
Int
)
(ids :
List
Name
)
(type? :
Option
Expr
)
(fmt :
Format
)
:
MetaM
Format
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
ppGoal
.
ppVars
(indent :
Int
)
(showLetValues :
Bool
)
(varNames :
List
Name
)
(prevType? :
Option
Expr
)
(fmt :
Format
)
(localDecl :
LocalDecl
)
:
MetaM
(
List
Name
×
Option
Expr
×
Format
)
Equations
One or more equations did not get rendered due to their size.
Instances For