File tree Expand file tree Collapse file tree 1 file changed +0
-23
lines changed
Expand file tree Collapse file tree 1 file changed +0
-23
lines changed Original file line number Diff line number Diff line change @@ -33,29 +33,6 @@ public meta section
3333
3434open Std (TreeMap)
3535
36- namespace Std.TreeMap
37-
38- -- This will be replaced by a `BEq` instance implemented in the standard library,
39- -- likely in Q4 2025.
40-
41- /-- Returns true if the two maps have the same size and the same keys and values
42- (with keys compared using the ordering, and values compared using `BEq`). -/
43- def beq {α β : Type *} [BEq β] {c : α → α → Ordering} (m₁ m₂ : TreeMap α β c) : Bool :=
44- m₁.size == m₂.size && Id.run do
45- -- This could be made more efficient by simultaneously traversing both maps.
46- for (k, v) in m₁ do
47- if let some v' := m₂[k]? then
48- if v != v' then
49- return false
50- else
51- return false
52- return true
53-
54- instance {α β : Type*} [BEq β] {c : α → α → Ordering} : BEq (TreeMap α β c) := ⟨beq⟩
55-
56- end Std.TreeMap
57-
58-
5936section
6037open Lean Elab Tactic Meta
6138
You can’t perform that action at this time.
0 commit comments