Equations
- Lean.Meta.DiscrTree.mkNoindexAnnotation e = Lean.mkAnnotation `noindex e
Instances For
Equations
- Lean.Meta.DiscrTree.hasNoindexAnnotation e = (Lean.annotation? `noindex e).isSome
Instances For
Equations
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- (Lean.Meta.DiscrTree.Key.lit v₁).lt (Lean.Meta.DiscrTree.Key.lit v₂) = decide (v₁ < v₂)
- (Lean.Meta.DiscrTree.Key.fvar n₁ a₁).lt (Lean.Meta.DiscrTree.Key.fvar n₂ a₂) = (n₁.name.quickLt n₂.name || n₁ == n₂ && decide (a₁ < a₂))
- (Lean.Meta.DiscrTree.Key.const n₁ a₁).lt (Lean.Meta.DiscrTree.Key.const n₂ a₂) = (n₁.quickLt n₂ || n₁ == n₂ && decide (a₁ < a₂))
- (Lean.Meta.DiscrTree.Key.proj s₁ i₁ a₁).lt (Lean.Meta.DiscrTree.Key.proj s₂ i₂ a₂) = (s₁.quickLt s₂ || s₁ == s₂ && decide (i₁ < i₂) || s₁ == s₂ && i₁ == i₂ && decide (a₁ < a₂))
- x✝¹.lt x✝ = decide (x✝¹.ctorIdx < x✝.ctorIdx)
Instances For
Equations
- Lean.Meta.DiscrTree.instLTKey = { lt := fun (a b : Lean.Meta.DiscrTree.Key) => a.lt b = true }
Equations
- Lean.Meta.DiscrTree.instDecidableLtKey a b = inferInstanceAs (Decidable (a.lt b = true))
Equations
- Lean.Meta.DiscrTree.Key.star.format = Std.Format.text "*"
- Lean.Meta.DiscrTree.Key.other.format = Std.Format.text "◾"
- (Lean.Meta.DiscrTree.Key.lit (Lean.Literal.natVal v)).format = Std.format v
- (Lean.Meta.DiscrTree.Key.lit (Lean.Literal.strVal v)).format = repr v
- (Lean.Meta.DiscrTree.Key.const k a).format = Std.format k
- (Lean.Meta.DiscrTree.Key.proj s i a).format = Std.format s ++ Std.Format.text "." ++ Std.format i
- (Lean.Meta.DiscrTree.Key.fvar k a).format = Std.format k.name
- Lean.Meta.DiscrTree.Key.arrow.format = Std.Format.text "∀"
Instances For
Equations
Equations
Equations
Helper function for converting an entry (i.e., Array Key) to the discrimination tree into
MessageData that is more user-friendly. We use this function to implement diagnostic information.
Equations
Instances For
@[deprecated Lean.Meta.DiscrTree.insertKeyValue (since := "2026-01-02")]
def
Lean.Meta.DiscrTree.insertCore
{α : Type}
[BEq α]
(d : DiscrTree α)
(keys : Array Key)
(v : α)
:
Equations
- d.insertCore keys v = d.insertKeyValue keys v