File tree Expand file tree Collapse file tree 1 file changed +8
-8
lines changed
Expand file tree Collapse file tree 1 file changed +8
-8
lines changed Original file line number Diff line number Diff line change @@ -517,18 +517,18 @@ Compares two hash maps using Boolean equality on keys and values.
517517Returns `true` if the maps contain the same key-value pairs, `false` otherwise.
518518-/
519519def beq [BEq α] [Hashable α] [LawfulBEq α] [∀ k, BEq (β k)] (m₁ m₂ : Raw α β) : Bool :=
520- if h : 0 < m₁.buckets.size ∧ 0 < m₂.buckets.size then
521- Raw₀.beq ⟨m₁, h.1 ⟩ ⟨m₂, h.2 ⟩
522- else
523- false
520+ if h : 0 < m₁.buckets.size ∧ 0 < m₂.buckets.size then
521+ Raw₀.beq ⟨m₁, h.1 ⟩ ⟨m₂, h.2 ⟩
522+ else
523+ false
524524
525525instance [BEq α] [Hashable α] [LawfulBEq α] [∀ k, BEq (β k)] : BEq (Raw α β) := ⟨beq⟩
526526
527527@[inherit_doc DHashMap.Raw.beq] def Const.beq {β : Type v} [BEq α] [Hashable α] [BEq β] (m₁ m₂ : Raw α (fun _ => β)) : Bool :=
528- if h : 0 < m₁.buckets.size ∧ 0 < m₂.buckets.size then
529- Raw₀.Const.beq ⟨m₁, h.1 ⟩ ⟨m₂, h.2 ⟩
530- else
531- false
528+ if h : 0 < m₁.buckets.size ∧ 0 < m₂.buckets.size then
529+ Raw₀.Const.beq ⟨m₁, h.1 ⟩ ⟨m₂, h.2 ⟩
530+ else
531+ false
532532
533533/--
534534Computes the difference of the given hash maps.
You can’t perform that action at this time.
0 commit comments