- byTarget : Lean.Meta.DiscrTree (Rule α)
- byHyp : Lean.Meta.DiscrTree (Rule α)
- unindexed : Lean.PHashSet (Rule α)
Instances For
Equations
- Aesop.instInhabitedIndex = { default := { byTarget := default, byHyp := default, unindexed := default } }
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Index.trace.traceArray
{α : Type}
[ToString (Rule α)]
(traceOpt : TraceOption)
(as : Array (Rule α))
:
Equations
- Aesop.Index.trace.traceArray traceOpt as = Array.forM (fun (r : String) => Lean.addTrace traceOpt.traceClass (Lean.toMessageData r)) (Array.map toString as).qsortOrd
Instances For
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.
Instances For
@[specialize #[]]
@[always_inline]
def
Aesop.Index.unindex.filterDiscrTree'
{α : Type}
(p : Rule α → Bool)
(unindexed : Lean.PHashSet (Rule α))
(t : Lean.Meta.DiscrTree (Rule α))
:
Lean.Meta.DiscrTree (Rule α) × Lean.PHashSet (Rule α)
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[specialize #[]]
def
Aesop.Index.applicableRules
{α : Type}
[Ord α]
(ri : Index α)
(goal : Lean.MVarId)
(include? : Rule α → Bool)
:
Lean.MetaM (Array (IndexMatchResult (Rule α)))
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[inline]
def
Aesop.Index.applicableRules.insertIndexMatchResults
{α : Type}
[Ord α]
(m : Lean.RBMap (Rule α) (Array IndexMatchLocation) Rule.compareByPriorityThenName)
(rs : Array (Rule α × Array IndexMatchLocation))
:
Equations
- One or more equations did not get rendered due to their size.