- ref : Lean.Syntax
- modifiers : Lean.Elab.Modifiers
- kind : Lean.Elab.DefKind
- shortDeclName : Lean.Name
- declName : Lean.Name
- binderIds : Array Lean.Syntax
- numParams : Nat
- type : Lean.Expr
- valueStx : Lean.Syntax
Equations
- One or more equations did not get rendered due to their size.
@[inline]
- usedFVarsMap : Lean.Elab.Term.MutualClosure.UsedFVarsMap
- modified : Bool
@[inline]
def
Lean.Elab.Term.MutualClosure.FixPoint.run
(letRecFVarIds : Array Lean.FVarId)
(usedFVarsMap : Lean.Elab.Term.MutualClosure.UsedFVarsMap)
:
Equations
- One or more equations did not get rendered due to their size.
@[inline]
- newLocalDecls : Array Lean.LocalDecl
- localDecls : Array Lean.LocalDecl
- newLetDecls : Array Lean.LocalDecl
- ref : Lean.Syntax
- localDecls : Array Lean.LocalDecl
- closed : Lean.Expr
- toLift : Lean.Elab.Term.LetRecToLift
@[inline]
def
Lean.Elab.Term.MutualClosure.insertReplacementForMainFns
(r : Lean.Elab.Term.MutualClosure.Replacement)
(sectionVars : Array Lean.Expr)
(mainHeaders : Array Lean.Elab.DefViewElabHeader)
(mainFVars : Array Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.MutualClosure.insertReplacementForLetRecs
(r : Lean.Elab.Term.MutualClosure.Replacement)
(letRecClosures : List Lean.Elab.Term.MutualClosure.LetRecClosure)
:
Equations
- Lean.Elab.Term.MutualClosure.insertReplacementForLetRecs r letRecClosures = List.foldl (fun r c => Std.RBMap.insert r c.toLift.fvarId c.closed) r letRecClosures
def
Lean.Elab.Term.MutualClosure.Replacement.apply
(r : Lean.Elab.Term.MutualClosure.Replacement)
(e : Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.MutualClosure.pushMain
(preDefs : Array Lean.Elab.PreDefinition)
(sectionVars : Array Lean.Expr)
(mainHeaders : Array Lean.Elab.DefViewElabHeader)
(mainVals : Array Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.MutualClosure.pushLetRecs
(preDefs : Array Lean.Elab.PreDefinition)
(letRecClosures : List Lean.Elab.Term.MutualClosure.LetRecClosure)
(kind : Lean.Elab.DefKind)
(modifiers : Lean.Elab.Modifiers)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.MutualClosure.getKindForLetRecs
(mainHeaders : Array Lean.Elab.DefViewElabHeader)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.MutualClosure.getModifiersForLetRecs
(mainHeaders : Array Lean.Elab.DefViewElabHeader)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.MutualClosure.main
(sectionVars : Array Lean.Expr)
(mainHeaders : Array Lean.Elab.DefViewElabHeader)
(mainFVars : Array Lean.Expr)
(mainVals : Array Lean.Expr)
(letRecsToLift : List Lean.Elab.Term.LetRecToLift)
:
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.
Remove auxiliary match discriminant let-declarations.
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.checkForHiddenUnivLevels
(allUserLevelNames : List Lean.Name)
(preDefs : Array Lean.Elab.PreDefinition)
:
Equations
- One or more equations did not get rendered due to their size.
partial def
Lean.Elab.Term.checkForHiddenUnivLevels.visitLevel
(allUserLevelNames : List Lean.Name)
(sTypes : Lean.CollectLevelParams.State)
(preDef : Lean.Elab.PreDefinition)
(u : Lean.Level)
:
partial def
Lean.Elab.Term.checkForHiddenUnivLevels.visit
(allUserLevelNames : List Lean.Name)
(sTypes : Lean.CollectLevelParams.State)
(preDef : Lean.Elab.PreDefinition)
(e : Lean.Expr)
:
def
Lean.Elab.Term.elabMutualDef
(vars : Array Lean.Expr)
(views : Array Lean.Elab.DefView)
(hints : Lean.Elab.TerminationHints)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.elabMutualDef.go
(vars : Array Lean.Expr)
(views : Array Lean.Elab.DefView)
(hints : Lean.Elab.TerminationHints)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.elabMutualDef.processDeriving
(views : Array Lean.Elab.DefView)
(headers : Array Lean.Elab.DefViewElabHeader)
:
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.