Skip to content

Commit

Permalink
Forward.Match: remove dead code
Browse files Browse the repository at this point in the history
  • Loading branch information
JLimperg committed Dec 2, 2024
1 parent 05d2cb2 commit 60b7e8f
Showing 1 changed file with 0 additions and 6 deletions.
6 changes: 0 additions & 6 deletions Aesop/Forward/Match.lean
Original file line number Diff line number Diff line change
Expand Up @@ -99,12 +99,6 @@ namespace ForwardRuleMatch
instance : ToMessageData ForwardRuleMatch where
toMessageData m := m!"{m.rule.name} {m.match.toMessageData m.rule}"

/-- Compare two queue entries by rule priority and rule name. Higher-priority
rules are considered less (since the queues are min-queues). -/
protected def compare (m₁ m₂ : ForwardRuleMatch) : Ordering :=
compare m₁.rule m₂.rule |>.then $
compare m₁.match m₂.match

/-- Fold over the hypotheses contained in a match. -/
def foldHypsM [Monad M] (f : σ → FVarId → M σ) (init : σ)
(m : ForwardRuleMatch) : M σ :=
Expand Down

0 comments on commit 60b7e8f

Please sign in to comment.