Skip to content

Commit e96006b

Browse files
committed
chore(Order/SuccPred/CompleteLinearOrder): spacing fixes (#19799)
1 parent c4c2823 commit e96006b

File tree

1 file changed

+24
-32
lines changed

1 file changed

+24
-32
lines changed

Mathlib/Order/SuccPred/CompleteLinearOrder.lean

Lines changed: 24 additions & 32 deletions
Original file line numberDiff line numberDiff line change
@@ -19,8 +19,7 @@ section ConditionallyCompleteLinearOrder
1919
variable [ConditionallyCompleteLinearOrder α] [Nonempty ι] {f : ι → α} {s : Set α} {x : α}
2020

2121
lemma csSup_mem_of_not_isSuccPrelimit
22-
(hne : s.Nonempty) (hbdd : BddAbove s) (hlim : ¬ IsSuccPrelimit (sSup s)) :
23-
sSup s ∈ s := by
22+
(hne : s.Nonempty) (hbdd : BddAbove s) (hlim : ¬ IsSuccPrelimit (sSup s)) : sSup s ∈ s := by
2423
obtain ⟨y, hy⟩ := not_forall_not.mp hlim
2524
obtain ⟨i, his, hi⟩ := exists_lt_of_lt_csSup hne hy.lt
2625
exact eq_of_le_of_not_lt (le_csSup hbdd his) (hy.2 hi) ▸ his
@@ -29,8 +28,7 @@ lemma csSup_mem_of_not_isSuccPrelimit
2928
alias csSup_mem_of_not_isSuccLimit := csSup_mem_of_not_isSuccPrelimit
3029

3130
lemma csInf_mem_of_not_isPredPrelimit
32-
(hne : s.Nonempty) (hbdd : BddBelow s) (hlim : ¬ IsPredPrelimit (sInf s)) :
33-
sInf s ∈ s := by
31+
(hne : s.Nonempty) (hbdd : BddBelow s) (hlim : ¬ IsPredPrelimit (sInf s)) : sInf s ∈ s := by
3432
obtain ⟨y, hy⟩ := not_forall_not.mp hlim
3533
obtain ⟨i, his, hi⟩ := exists_lt_of_csInf_lt hne hy.lt
3634
exact eq_of_le_of_not_lt (csInf_le hbdd his) (hy.2 · hi) ▸ his
@@ -39,17 +37,15 @@ lemma csInf_mem_of_not_isPredPrelimit
3937
alias csInf_mem_of_not_isPredLimit := csInf_mem_of_not_isPredPrelimit
4038

4139
lemma exists_eq_ciSup_of_not_isSuccPrelimit
42-
(hf : BddAbove (Set.range f)) (hf' : ¬ IsSuccPrelimit (⨆ i, f i)) :
43-
∃ i, f i = ⨆ i, f i :=
44-
csSup_mem_of_not_isSuccPrelimit (Set.range_nonempty f) hf hf'
40+
(hf : BddAbove (range f)) (hf' : ¬ IsSuccPrelimit (⨆ i, f i)) : ∃ i, f i = ⨆ i, f i :=
41+
csSup_mem_of_not_isSuccPrelimit (range_nonempty f) hf hf'
4542

4643
@[deprecated exists_eq_ciSup_of_not_isSuccPrelimit (since := "2024-09-05")]
4744
alias exists_eq_ciSup_of_not_isSuccLimit := exists_eq_ciSup_of_not_isSuccPrelimit
4845

4946
lemma exists_eq_ciInf_of_not_isPredPrelimit
50-
(hf : BddBelow (Set.range f)) (hf' : ¬ IsPredPrelimit (⨅ i, f i)) :
51-
∃ i, f i = ⨅ i, f i :=
52-
csInf_mem_of_not_isPredPrelimit (Set.range_nonempty f) hf hf'
47+
(hf : BddBelow (range f)) (hf' : ¬ IsPredPrelimit (⨅ i, f i)) : ∃ i, f i = ⨅ i, f i :=
48+
csInf_mem_of_not_isPredPrelimit (range_nonempty f) hf hf'
5349

5450
@[deprecated exists_eq_ciInf_of_not_isPredPrelimit (since := "2024-09-05")]
5551
alias exists_eq_ciInf_of_not_isPredLimit := exists_eq_ciInf_of_not_isPredPrelimit
@@ -69,15 +65,15 @@ lemma IsGLB.mem_of_nonempty_of_not_isPredPrelimit
6965
alias IsGLB.mem_of_nonempty_of_not_isPredLimit := IsGLB.mem_of_nonempty_of_not_isPredPrelimit
7066

7167
lemma IsLUB.exists_of_nonempty_of_not_isSuccPrelimit
72-
(hf : IsLUB (Set.range f) x) (hx : ¬ IsSuccPrelimit x) :
73-
∃ i, f i = x := hf.mem_of_nonempty_of_not_isSuccPrelimit (Set.range_nonempty f) hx
68+
(hf : IsLUB (range f) x) (hx : ¬ IsSuccPrelimit x) : ∃ i, f i = x :=
69+
hf.mem_of_nonempty_of_not_isSuccPrelimit (range_nonempty f) hx
7470

7571
@[deprecated IsLUB.exists_of_nonempty_of_not_isSuccPrelimit (since := "2024-09-05")]
7672
alias IsLUB.exists_of_nonempty_of_not_isSuccLimit := IsLUB.exists_of_nonempty_of_not_isSuccPrelimit
7773

7874
lemma IsGLB.exists_of_nonempty_of_not_isPredPrelimit
79-
(hf : IsGLB (Set.range f) x) (hx : ¬ IsPredPrelimit x) :
80-
∃ i, f i = x := hf.mem_of_nonempty_of_not_isPredPrelimit (Set.range_nonempty f) hx
75+
(hf : IsGLB (range f) x) (hx : ¬ IsPredPrelimit x) : ∃ i, f i = x :=
76+
hf.mem_of_nonempty_of_not_isPredPrelimit (range_nonempty f) hx
8177

8278
@[deprecated IsGLB.exists_of_nonempty_of_not_isPredPrelimit (since := "2024-09-05")]
8379
alias IsGLB.exists_of_nonempty_of_not_isPredLimit := IsGLB.exists_of_nonempty_of_not_isPredPrelimit
@@ -110,9 +106,8 @@ variable [ConditionallyCompleteLinearOrderBot α] {f : ι → α} {s : Set α} {
110106

111107
/-- See `csSup_mem_of_not_isSuccPrelimit` for the `ConditionallyCompleteLinearOrder` version. -/
112108
lemma csSup_mem_of_not_isSuccPrelimit'
113-
(hbdd : BddAbove s) (hlim : ¬ IsSuccPrelimit (sSup s)) :
114-
sSup s ∈ s := by
115-
obtain (rfl|hs) := s.eq_empty_or_nonempty
109+
(hbdd : BddAbove s) (hlim : ¬ IsSuccPrelimit (sSup s)) : sSup s ∈ s := by
110+
obtain rfl | hs := s.eq_empty_or_nonempty
116111
· simp [isSuccPrelimit_bot] at hlim
117112
· exact csSup_mem_of_not_isSuccPrelimit hs hbdd hlim
118113

@@ -122,24 +117,23 @@ alias csSup_mem_of_not_isSuccLimit' := csSup_mem_of_not_isSuccPrelimit'
122117
/-- See `exists_eq_ciSup_of_not_isSuccPrelimit` for the
123118
`ConditionallyCompleteLinearOrder` version. -/
124119
lemma exists_eq_ciSup_of_not_isSuccPrelimit'
125-
(hf : BddAbove (Set.range f)) (hf' : ¬ IsSuccPrelimit (⨆ i, f i)) :
126-
∃ i, f i = ⨆ i, f i :=
120+
(hf : BddAbove (range f)) (hf' : ¬ IsSuccPrelimit (⨆ i, f i)) : ∃ i, f i = ⨆ i, f i :=
127121
csSup_mem_of_not_isSuccPrelimit' hf hf'
128122

129123
@[deprecated exists_eq_ciSup_of_not_isSuccPrelimit' (since := "2024-09-05")]
130124
alias exists_eq_ciSup_of_not_isSuccLimit' := exists_eq_ciSup_of_not_isSuccPrelimit'
131125

132-
lemma IsLUB.mem_of_not_isSuccPrelimit (hs : IsLUB s x) (hx : ¬ IsSuccPrelimit x) :
133-
x ∈ s := by
134-
obtain (rfl|hs') := s.eq_empty_or_nonempty
126+
lemma IsLUB.mem_of_not_isSuccPrelimit (hs : IsLUB s x) (hx : ¬ IsSuccPrelimit x) : x ∈ s := by
127+
obtain rfl | hs' := s.eq_empty_or_nonempty
135128
· simp [show x = ⊥ by simpa using hs, isSuccPrelimit_bot] at hx
136129
· exact hs.mem_of_nonempty_of_not_isSuccPrelimit hs' hx
137130

138131
@[deprecated IsLUB.mem_of_not_isSuccPrelimit (since := "2024-09-05")]
139132
alias IsLUB.mem_of_not_isSuccLimit := IsLUB.mem_of_not_isSuccPrelimit
140133

141-
lemma IsLUB.exists_of_not_isSuccPrelimit (hf : IsLUB (Set.range f) x) (hx : ¬ IsSuccPrelimit x) :
142-
∃ i, f i = x := hf.mem_of_not_isSuccPrelimit hx
134+
lemma IsLUB.exists_of_not_isSuccPrelimit (hf : IsLUB (range f) x) (hx : ¬ IsSuccPrelimit x) :
135+
∃ i, f i = x :=
136+
hf.mem_of_not_isSuccPrelimit hx
143137

144138
@[deprecated IsLUB.exists_of_not_isSuccPrelimit (since := "2024-09-05")]
145139
alias IsLUB.exists_of_not_isSuccLimit := IsLUB.exists_of_not_isSuccPrelimit
@@ -175,17 +169,15 @@ end ConditionallyCompleteLinearOrderBot
175169
section CompleteLinearOrder
176170
variable [CompleteLinearOrder α] {s : Set α} {f : ι → α} {x : α}
177171

178-
lemma sSup_mem_of_not_isSuccPrelimit (hlim : ¬ IsSuccPrelimit (sSup s)) :
179-
sSup s ∈ s := by
172+
lemma sSup_mem_of_not_isSuccPrelimit (hlim : ¬ IsSuccPrelimit (sSup s)) : sSup s ∈ s := by
180173
obtain ⟨y, hy⟩ := not_forall_not.mp hlim
181174
obtain ⟨i, his, hi⟩ := lt_sSup_iff.mp hy.lt
182175
exact eq_of_le_of_not_lt (le_sSup his) (hy.2 hi) ▸ his
183176

184177
@[deprecated sSup_mem_of_not_isSuccPrelimit (since := "2024-09-05")]
185178
alias sSup_mem_of_not_isSuccLimit := sSup_mem_of_not_isSuccPrelimit
186179

187-
lemma sInf_mem_of_not_isPredPrelimit (hlim : ¬ IsPredPrelimit (sInf s)) :
188-
sInf s ∈ s := by
180+
lemma sInf_mem_of_not_isPredPrelimit (hlim : ¬ IsPredPrelimit (sInf s)) : sInf s ∈ s := by
189181
obtain ⟨y, hy⟩ := not_forall_not.mp hlim
190182
obtain ⟨i, his, hi⟩ := sInf_lt_iff.mp hy.lt
191183
exact eq_of_le_of_not_lt (sInf_le his) (hy.2 · hi) ▸ his
@@ -207,15 +199,15 @@ lemma exists_eq_iInf_of_not_isPredPrelimit (hf : ¬ IsPredPrelimit (⨅ i, f i))
207199
@[deprecated exists_eq_iInf_of_not_isPredPrelimit (since := "2024-09-05")]
208200
alias exists_eq_iInf_of_not_isPredLimit := exists_eq_iInf_of_not_isPredPrelimit
209201

210-
lemma IsGLB.mem_of_not_isPredPrelimit (hs : IsGLB s x) (hx : ¬ IsPredPrelimit x) :
211-
x ∈ s :=
202+
lemma IsGLB.mem_of_not_isPredPrelimit (hs : IsGLB s x) (hx : ¬ IsPredPrelimit x) : x ∈ s :=
212203
hs.sInf_eq ▸ sInf_mem_of_not_isPredPrelimit (hs.sInf_eq ▸ hx)
213204

214205
@[deprecated IsGLB.mem_of_not_isPredPrelimit (since := "2024-09-05")]
215206
alias IsGLB.mem_of_not_isPredLimit := IsGLB.mem_of_not_isPredPrelimit
216207

217-
lemma IsGLB.exists_of_not_isPredPrelimit (hf : IsGLB (Set.range f) x) (hx : ¬ IsPredPrelimit x) :
218-
∃ i, f i = x := hf.mem_of_not_isPredPrelimit hx
208+
lemma IsGLB.exists_of_not_isPredPrelimit (hf : IsGLB (range f) x) (hx : ¬ IsPredPrelimit x) :
209+
∃ i, f i = x :=
210+
hf.mem_of_not_isPredPrelimit hx
219211

220212
@[deprecated IsGLB.exists_of_not_isPredPrelimit (since := "2024-09-05")]
221213
alias IsGLB.exists_of_not_isPredLimit := IsGLB.exists_of_not_isPredPrelimit

0 commit comments

Comments
 (0)