@@ -138,24 +138,23 @@ theorem atTop_hasAntitoneBasis_of_archimedean [OrderedSemiring R] [Archimedean R
138
138
(atTop : Filter R).HasAntitoneBasis fun n : ℕ => Ici n :=
139
139
hasAntitoneBasis_atTop.comp_mono Nat.mono_cast tendsto_natCast_atTop_atTop
140
140
141
- theorem atTop_hasCountableBasis_of_archimedean [StrictOrderedSemiring R] [Archimedean R] :
141
+ theorem atTop_hasCountableBasis_of_archimedean [OrderedSemiring R] [Archimedean R] :
142
142
(atTop : Filter R).HasCountableBasis (fun _ : ℕ => True) fun n => Ici n :=
143
143
⟨atTop_hasAntitoneBasis_of_archimedean.1 , to_countable _⟩
144
144
145
- -- Porting note (#11215): TODO: generalize to a `StrictOrderedRing`
146
- theorem atBot_hasCountableBasis_of_archimedean [LinearOrderedRing R] [Archimedean R] :
147
- (atBot : Filter R).HasCountableBasis (fun _ : ℤ => True) fun m => Iic m :=
148
- { countable := to_countable _
149
- toHasBasis :=
150
- atBot_basis.to_hasBasis
151
- (fun x _ => let ⟨m, hm⟩ := exists_int_lt x; ⟨m, trivial, Iic_subset_Iic.2 hm.le⟩)
152
- fun m _ => ⟨m, trivial, Subset.rfl⟩ }
145
+ theorem atBot_hasCountableBasis_of_archimedean [OrderedRing R] [Archimedean R] :
146
+ (atBot : Filter R).HasCountableBasis (fun _ : ℤ => True) fun m => Iic m where
147
+ countable := to_countable _
148
+ toHasBasis :=
149
+ atBot_basis.to_hasBasis
150
+ (fun x _ => let ⟨m, hm⟩ := exists_int_le x; ⟨m, trivial, Iic_subset_Iic.2 hm⟩)
151
+ fun m _ => ⟨m, trivial, Subset.rfl⟩
153
152
154
- instance (priority := 100 ) atTop_isCountablyGenerated_of_archimedean [StrictOrderedSemiring R]
153
+ instance (priority := 100 ) atTop_isCountablyGenerated_of_archimedean [OrderedSemiring R]
155
154
[Archimedean R] : (atTop : Filter R).IsCountablyGenerated :=
156
155
atTop_hasCountableBasis_of_archimedean.isCountablyGenerated
157
156
158
- instance (priority := 100 ) atBot_isCountablyGenerated_of_archimedean [LinearOrderedRing R]
157
+ instance (priority := 100 ) atBot_isCountablyGenerated_of_archimedean [OrderedRing R]
159
158
[Archimedean R] : (atBot : Filter R).IsCountablyGenerated :=
160
159
atBot_hasCountableBasis_of_archimedean.isCountablyGenerated
161
160
0 commit comments