- unindexed : IndexingMode
- target (keys : Array Lean.Meta.DiscrTree.Key) : IndexingMode
- hyps (keys : Array Lean.Meta.DiscrTree.Key) : IndexingMode
- or (imodes : Array IndexingMode) : IndexingMode
Instances For
Equations
Equations
Equations
- Aesop.IndexingMode.targetMatchingConclusion type = do let path ← Aesop.getConclusionDiscrTreeKeys type pure (Aesop.IndexingMode.target path)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
The source of a rule match reported by the index. We assume that only IndexMatchLocations belonging to the same goal are equated or compared.
- none : IndexMatchLocation
- target : IndexMatchLocation
- hyp (ldecl : Lean.LocalDecl) : IndexMatchLocation
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.
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.
A rule that, according to the index, should be applied to the current goal. In addition to the rule, this data structure contains information about how the rule should be applied. For example, if the rule has rule patterns, we report the substitutions obtained by matching the rule patterns against the current goal.
- rule : α
The rule that should be applied.
- locations : Array IndexMatchLocation
Goal locations where the rule matched. The rule's
indexingModedetermines which locations can be contained in this set. The array contains no duplicates. - patternSubsts? : Option (Array Substitution)
Pattern substitutions for this rule that were found in the goal.
noneiff the rule doesn't have a pattern. The array contains no duplicates.
Instances For
Equations
Equations
Instances For
Equations
- Aesop.IndexMatchResult.instOrd = { compare := fun (r s : Aesop.IndexMatchResult α) => compare r.rule s.rule }
Equations
Equations
- Aesop.IndexMatchResult.instToMessageData = { toMessageData := fun (r : Aesop.IndexMatchResult α) => Lean.toMessageData r.rule }