Skip to content

Commit

Permalink
.
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Jan 6, 2025
1 parent f93b006 commit 86818a7
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Batteries/Data/RBMap/WF.lean
Original file line number Diff line number Diff line change
Expand Up @@ -124,7 +124,7 @@ theorem setBlack_idem {t : RBNode α} : t.setBlack.setBlack = t.setBlack := by c
protected theorem All.ins {x : α} {t : RBNode α}
(h₁ : p x) (h₂ : t.All p) : (ins cmp x t).All p := by
induction t <;> unfold ins <;> try simp [*]
split <;> cases ‹_=_› <;> split <;> simp at h₂ <;> simp [*]
split <;> cases ‹_ = _› <;> split <;> simp at h₂ <;> simp [*]

/-- The `ins` function preserves the ordering invariants. -/
protected theorem Ordered.ins : ∀ {t : RBNode α}, t.Ordered cmp → (ins cmp x t).Ordered cmp
Expand Down

0 comments on commit 86818a7

Please sign in to comment.