Documentation
Lean
.
Elab
.
LetRec
Search
return to top
source
Imports
Lean.Elab.Attributes
Lean.Elab.Binders
Lean.Elab.DeclModifiers
Lean.Elab.DeclarationRange
Lean.Elab.SyntheticMVars
Imported by
Lean
.
Elab
.
Term
.
LetRecDeclView
Lean
.
Elab
.
Term
.
LetRecView
Lean
.
Elab
.
Term
.
elabLetRec
source
structure
Lean
.
Elab
.
Term
.
LetRecDeclView
:
Type
ref :
Syntax
attrs :
Array
Attribute
shortDeclName :
Name
declName :
Name
binderIds :
Array
Syntax
type :
Expr
mvar :
Expr
valStx :
Syntax
termination :
TerminationHints
Instances For
source
structure
Lean
.
Elab
.
Term
.
LetRecView
:
Type
decls :
Array
LetRecDeclView
body :
Syntax
Instances For
source
def
Lean
.
Elab
.
Term
.
elabLetRec
:
TermElab
Equations
One or more equations did not get rendered due to their size.
Instances For