Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit c985ae9

Browse files
committed
chore(topology/order/basic): generalise frontier_Icc (#18571)
1 parent f24cc28 commit c985ae9

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/topology/order/basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -2132,9 +2132,9 @@ by simp [frontier, closure_Iio' ha, Iic_diff_Iio, Icc_self]
21322132
lemma frontier_Iio [no_min_order α] {a : α} : frontier (Iio a) = {a} :=
21332133
frontier_Iio' nonempty_Iio
21342134

2135-
@[simp] lemma frontier_Icc [no_min_order α] [no_max_order α] {a b : α} (h : a < b) :
2135+
@[simp] lemma frontier_Icc [no_min_order α] [no_max_order α] {a b : α} (h : a b) :
21362136
frontier (Icc a b) = {a, b} :=
2137-
by simp [frontier, le_of_lt h, Icc_diff_Ioo_same]
2137+
by simp [frontier, h, Icc_diff_Ioo_same]
21382138

21392139
@[simp] lemma frontier_Ioo {a b : α} (h : a < b) : frontier (Ioo a b) = {a, b} :=
21402140
by rw [frontier, closure_Ioo h.ne, interior_Ioo, Icc_diff_Ioo_same h.le]

0 commit comments

Comments
 (0)