Skip to content

Commit 179addf

Browse files
committed
chore: fix indentation
1 parent d0e16d9 commit 179addf

File tree

1 file changed

+8
-8
lines changed

1 file changed

+8
-8
lines changed

src/Std/Data/DHashMap/Raw.lean

Lines changed: 8 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -517,18 +517,18 @@ Compares two hash maps using Boolean equality on keys and values.
517517
Returns `true` if the maps contain the same key-value pairs, `false` otherwise.
518518
-/
519519
def 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

525525
instance [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
/--
534534
Computes the difference of the given hash maps.

0 commit comments

Comments
 (0)