Skip to content

Commit

Permalink
Util.UnorderedArraySet: remove quadratic BEq instance (#162)
Browse files Browse the repository at this point in the history
  • Loading branch information
JLimperg authored Sep 29, 2024
1 parent a895713 commit 50aaaf7
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 4 deletions.
1 change: 1 addition & 0 deletions Aesop/Tracing.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,7 @@ Authors: Jannis Limperg
-/

import Aesop.Util.Basic
import Batteries.Data.Array.Basic
import Lean.Elab.Term
import Lean.Meta.Tactic.Simp

Expand Down
4 changes: 0 additions & 4 deletions Aesop/Util/UnorderedArraySet.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2021 Jannis Limperg. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jannis Limperg
-/
import Batteries.Data.Array.Basic
import Batteries.Data.Array.Merge
import Lean.Message

Expand Down Expand Up @@ -131,9 +130,6 @@ def all (p : α → Bool) (s : UnorderedArraySet α) (start := 0) (stop := s.siz
Bool :=
s.rep.all p start stop

instance : BEq (UnorderedArraySet α) where
beq s t := s.rep.equalSet t.rep

instance [ToString α] : ToString (UnorderedArraySet α) where
toString s := toString s.rep

Expand Down

0 comments on commit 50aaaf7

Please sign in to comment.