Instances For
Equations
Equations
- Lean.Elab.instBEqDefKind.beq x✝ y✝ = (x✝.ctorIdx == y✝.ctorIdx)
Instances For
Equations
Header elaboration data of a DefView.
- shortDeclName : NameShort name. Recall that all declarations in Lean 4 are potentially recursive. We use shortDeclNameto refer to them atvalueStx, and other declarations in the same mutual block.
- declName : NameFull name for this declaration. This is the name that will be added to the Environment.
- Universe level parameter names explicitly provided by the user. 
- Syntax objects for the binders occurring before - :, we use them to populate the- InfoTreewhen elaborating- valueStx.
- numParams : NatNumber of parameters before :, it also includes auto-implicit parameters automatically added by Lean.
- type : ExprType including parameters. 
Instances For
Equations
Instances For
Snapshot after processing of a definition body.
- state : Term.SavedStateState after elaboration. 
- value : ExprElaboration result. 
- moreSnaps : Array (Language.SnapshotTask Language.SnapshotTree)Untyped snapshots from logSnapshotTask, saved at this level for cancellation.
Instances For
Equations
- Lean.Elab.instToSnapshotTreeBodyProcessedSnapshot = { toSnapshotTree := fun (s : Lean.Elab.BodyProcessedSnapshot) => { element := s.toSnapshot, children := s.moreSnaps } }
Snapshot after elaboration of a definition header.
- view : DefViewElabHeaderDataElaboration results. 
- state : Term.SavedStateResulting elaboration state, including any environment additions. 
- Syntax of top-level tactic block if any, for checking reuse of - tacSnap?.
- tacSnap? : Option (Language.SnapshotTask Tactic.TacticParsedSnapshot)Incremental execution of main tactic block, if any. 
- bodyStx : SyntaxSyntax of definition body, for checking reuse of bodySnap.
- bodySnap : Language.SnapshotTask (Option BodyProcessedSnapshot)Result of body elaboration. 
- moreSnaps : Array (Language.SnapshotTask Language.SnapshotTree)Untyped snapshots from logSnapshotTask, saved at this level for cancellation.
Instances For
Equations
- One or more equations did not get rendered due to their size.
State before elaboration of a mutual definition.
- fullHeaderRef : SyntaxUnstructured syntax object comprising the full "header" of the definition from the modifiers (incl. docstring) up to the value, used for determining header elaboration reuse. 
- headerProcessedSnap : Language.SnapshotTask (Option HeaderProcessedSnapshot)Elaboration result, unless fatal exception occurred. 
Instances For
Snapshot after syntax tree has been split into separate mutual def headers.
- Definitions of this mutual block. 
Instances For
Equations
- One or more equations did not get rendered due to their size.
- kind : DefKind
- ref : Syntax
- headerRef : SyntaxAn unstructured syntax object that comprises the "header" of the definition, i.e. everything up to the value. Used as a more specific ref for header elaboration. 
- modifiers : Modifiers
- declId : Syntax
- binders : Syntax
- value : Syntax
- The docstring, if present, and whether it's Verso 
- headerSnap? : Option (Language.SnapshotBundle (Option HeaderProcessedSnapshot))Snapshot for incremental processing of this definition. Invariant: If the bundle's old?is set, then elaboration of the header is guaranteed to result in the same elaboration result and state, i.e. reuse is possible.
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- view.isInstance = view.modifiers.attrs.any fun (attr : Lean.Elab.Attribute) => attr.name == `instance
Instances For
Prepends the defeq attribute, removing existing ones if there are any
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.
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.
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.
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.