A (potentially recursive) definition. The elaborator converts it into Kernel definitions using many different strategies.
- ref : Lean.Syntax
- kind : Lean.Elab.DefKind
- modifiers : Lean.Elab.Modifiers
- declName : Lake.Name
- type : Lean.Expr
- value : Lean.Expr
- termination : Lean.Elab.WF.TerminationHints
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.fixLevelParams
(preDefs : Array Lean.Elab.PreDefinition)
(scopeLevelNames : List Lake.Name)
(allUserLevelNames : List Lake.Name)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.applyAttributesOf
(preDefs : Array Lean.Elab.PreDefinition)
(applicationTime : Lean.AttributeApplicationTime)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Auxiliary method for (temporarily) adding pre definition as an axiom
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.addAndCompileNonRec
(preDef : Lean.Elab.PreDefinition)
(all : optParam (List Lake.Name) [preDef.declName])
 :
Equations
- Lean.Elab.addAndCompileNonRec preDef all = Lean.Elab.addNonRecAux preDef true all
Instances For
def
Lean.Elab.addNonRec
(preDef : Lean.Elab.PreDefinition)
(applyAttrAfterCompilation : optParam Bool true)
(all : optParam (List Lake.Name) [preDef.declName])
 :
Equations
- Lean.Elab.addNonRec preDef applyAttrAfterCompilation all = Lean.Elab.addNonRecAux preDef false all applyAttrAfterCompilation
Instances For
Eliminate recursive application annotations containing syntax. These annotations are used by the well-founded recursion module to produce better error messages.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.addAndCompileUnsafe
(preDefs : Array Lean.Elab.PreDefinition)
(safety : optParam Lean.DefinitionSafety Lean.DefinitionSafety.unsafe)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.