Documentation

Lean.Meta.DiscrTree

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.
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
Equations
  • Lean.Meta.DiscrTree.instToFormatTrie = { format := Lean.Meta.DiscrTree.Trie.format }
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • Lean.Meta.DiscrTree.instToFormatDiscrTree = { format := Lean.Meta.DiscrTree.format }
Equations

whnf for the discrimination tree module

Equations
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.

Find values that match e in d.

Equations

Similar to getMatch, but returns solutions that are prefixes of e. We store the number of ignored arguments in the result.

Equations
  • One or more equations did not get rendered due to their size.
partial def Lean.Meta.DiscrTree.getMatchWithExtra.go {α : Type} (d : Lean.Meta.DiscrTree α) (e : Lean.Expr) (numExtra : Nat) (result : Array (α × Nat)) :
Equations
  • One or more equations did not get rendered due to their size.
partial def Lean.Meta.DiscrTree.getUnify.process {α : Type} (skip : Nat) (todo : Array Lean.Expr) (c : Lean.Meta.DiscrTree.Trie α) (result : Array α) :