@@ -195,18 +195,20 @@ end Image
195
195
196
196
section sequence
197
197
198
- variable {π : Type *} [NormedField π] [NontriviallyNormedField π] [AddCommGroup E] [Module π E]
199
- [Module π E] [TopologicalSpace E] [ContinuousSMul π E]
200
-
201
- theorem IsVonNBounded.smul_tendsto_zero {S : Set E} {Ξ΅ : ΞΉ β π} {x : ΞΉ β E} {l : Filter ΞΉ}
198
+ theorem IsVonNBounded.smul_tendsto_zero [NormedField π]
199
+ [AddCommGroup E] [Module π E] [TopologicalSpace E]
200
+ {S : Set E} {Ξ΅ : ΞΉ β π} {x : ΞΉ β E} {l : Filter ΞΉ}
202
201
(hS : IsVonNBounded π S) (hxS : βαΆ n in l, x n β S) (hΞ΅ : Tendsto Ξ΅ l (π 0 )) :
203
202
Tendsto (Ξ΅ β’ x) l (π 0 ) :=
204
203
(hS.tendsto_smallSets_nhds.comp hΞ΅).of_smallSets <| hxS.mono fun _ β¦ smul_mem_smul_set
205
204
206
- theorem isVonNBounded_of_smul_tendsto_zero {Ξ΅ : ΞΉ β π} {l : Filter ΞΉ} [l.NeBot]
205
+ variable [NontriviallyNormedField π]
206
+ [AddCommGroup E] [Module π E] [TopologicalSpace E] [ContinuousSMul π E]
207
+
208
+ theorem isVonNBounded_of_smul_tendsto_zero {Ξ΅ : ΞΉ β π} {l : Filter ΞΉ} [l.NeBot]
207
209
(hΞ΅ : βαΆ n in l, Ξ΅ n β 0 ) {S : Set E}
208
- (H : β x : ΞΉ β E, (β n, x n β S) β Tendsto (Ξ΅ β’ x) l (π 0 )) : IsVonNBounded π S := by
209
- rw [(nhds_basis_balanced π E).isVonNBounded_iff]
210
+ (H : β x : ΞΉ β E, (β n, x n β S) β Tendsto (Ξ΅ β’ x) l (π 0 )) : IsVonNBounded π S := by
211
+ rw [(nhds_basis_balanced π E).isVonNBounded_iff]
210
212
by_contra! H'
211
213
rcases H' with β¨V, β¨hV, hVbβ©, hVSβ©
212
214
have : βαΆ n in l, β x : S, Ξ΅ n β’ (x : E) β V := by
@@ -227,9 +229,9 @@ theorem isVonNBounded_of_smul_tendsto_zero {Ξ΅ : ΞΉ β π} {l : Filter ΞΉ} [l
227
229
if and only if for any sequence `x : β β S`, `Ξ΅ β’ x` tends to 0. This actually works for any
228
230
indexing type `ΞΉ`, but in the special case `ΞΉ = β` we get the important fact that convergent
229
231
sequences fully characterize bounded sets. -/
230
- theorem isVonNBounded_iff_smul_tendsto_zero {Ξ΅ : ΞΉ β π } {l : Filter ΞΉ} [l.NeBot]
232
+ theorem isVonNBounded_iff_smul_tendsto_zero {Ξ΅ : ΞΉ β π } {l : Filter ΞΉ} [l.NeBot]
231
233
(hΞ΅ : Tendsto Ξ΅ l (π[β ] 0 )) {S : Set E} :
232
- IsVonNBounded π S β β x : ΞΉ β E, (β n, x n β S) β Tendsto (Ξ΅ β’ x) l (π 0 ) :=
234
+ IsVonNBounded π S β β x : ΞΉ β E, (β n, x n β S) β Tendsto (Ξ΅ β’ x) l (π 0 ) :=
233
235
β¨fun hS x hxS => hS.smul_tendsto_zero (eventually_of_forall hxS) (le_trans hΞ΅ nhdsWithin_le_nhds),
234
236
isVonNBounded_of_smul_tendsto_zero (by exact hΞ΅ self_mem_nhdsWithin)β©
235
237
0 commit comments