def
Lean.Elab.Term.Quotation.resolveSectionVariable
(sectionVars : Lean.NameMap Lean.Name)
(id : Lean.Name)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.Quotation.resolveSectionVariable.loop
(sectionVars : Lean.NameMap Lean.Name)
(extractionResult : Lean.MacroScopesView)
:
Equations
- One or more equations did not get rendered due to their size.
- Lean.Elab.Term.Quotation.resolveSectionVariable.loop sectionVars extractionResult _fun_discr _fun_discr = []
Transform sequence of pushes and appends into acceptable code
Equations
- Lean.Elab.Term.Quotation.ArrayStxBuilder.build _fun_discr = match _fun_discr with | Sum.inl elems => Lean.quote `term elems | Sum.inr arr => arr
def
Lean.Elab.Term.Quotation.ArrayStxBuilder.push
(b : Lean.Elab.Term.Quotation.ArrayStxBuilder)
(elem : Lean.Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Term.Quotation.ArrayStxBuilder.append
(b : Lean.Elab.Term.Quotation.ArrayStxBuilder)
(arr : Lean.Syntax)
(appendName : optParam Lean.Name `Array.append)
:
Equations
- Lean.Elab.Term.Quotation.ArrayStxBuilder.append b arr appendName = Sum.inr (Lean.Syntax.mkCApp appendName #[Lean.Elab.Term.Quotation.ArrayStxBuilder.build b, { raw := arr }])
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.
Equations
- One or more equations did not get rendered due to their size.
- unconditional: Lean.Elab.Term.Quotation.HeadCheck
- shape: List Lean.SyntaxNodeKind → Option Nat → Lean.Elab.Term.Quotation.HeadCheck
- slice: Nat → Nat → Lean.Elab.Term.Quotation.HeadCheck
- other: Lean.Syntax → Lean.Elab.Term.Quotation.HeadCheck
In a single match step, we match the first discriminant against the "head" of the first pattern of the first
alternative. This datatype describes what kind of check this involves, which helps other patterns decide if
they are covered by the same check and don't have to be checked again (see also MatchResult
).
- covered: (Lean.Elab.Term.Quotation.Alt → Lean.Elab.TermElabM Lean.Elab.Term.Quotation.Alt) → Bool → Lean.Elab.Term.Quotation.MatchResult
- uncovered: Lean.Elab.Term.Quotation.MatchResult
- undecided: Lean.Elab.Term.Quotation.MatchResult
Describe whether a pattern is covered by a head check (induced by the pattern itself or a different pattern).
- doMatch : (List Lean.Term → Lean.Elab.TermElabM Lean.Term) → Lean.Elab.TermElabM Lean.Term → Lean.Elab.TermElabM Lean.Term
All necessary information on a pattern head.
Equations
- One or more equations did not get rendered due to their size.
Syntactic pattern match. Matches a Syntax
value against quotations, pattern variables, or _
.