Skip to content

Commit 56b98b2

Browse files
urkudbjoernkjoshanssen
authored andcommitted
chore(LocallyConvex/Bounded): rename variables (#15289)
Instead of introducing a normed field `π•œ` and a nontrivially normed field `𝕝`, prove a theorem for a normed field, then assume that `π•œ` is a nontrivially normed field.
1 parent 6ceede3 commit 56b98b2

File tree

1 file changed

+11
-9
lines changed

1 file changed

+11
-9
lines changed

β€ŽMathlib/Analysis/LocallyConvex/Bounded.lean

+11-9
Original file line numberDiff line numberDiff line change
@@ -195,18 +195,20 @@ end Image
195195

196196
section sequence
197197

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 ΞΉ}
202201
(hS : IsVonNBounded π•œ S) (hxS : βˆ€αΆ  n in l, x n ∈ S) (hΞ΅ : Tendsto Ξ΅ l (𝓝 0)) :
203202
Tendsto (Ξ΅ β€’ x) l (𝓝 0) :=
204203
(hS.tendsto_smallSets_nhds.comp hΞ΅).of_smallSets <| hxS.mono fun _ ↦ smul_mem_smul_set
205204

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]
207209
(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]
210212
by_contra! H'
211213
rcases H' with ⟨V, ⟨hV, hVb⟩, hVS⟩
212214
have : βˆ€αΆ  n in l, βˆƒ x : S, Ξ΅ n β€’ (x : E) βˆ‰ V := by
@@ -227,9 +229,9 @@ theorem isVonNBounded_of_smul_tendsto_zero {Ξ΅ : ΞΉ β†’ 𝕝} {l : Filter ΞΉ} [l
227229
if and only if for any sequence `x : β„• β†’ S`, `Ξ΅ β€’ x` tends to 0. This actually works for any
228230
indexing type `ΞΉ`, but in the special case `ΞΉ = β„•` we get the important fact that convergent
229231
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]
231233
(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) :=
233235
⟨fun hS x hxS => hS.smul_tendsto_zero (eventually_of_forall hxS) (le_trans hΡ nhdsWithin_le_nhds),
234236
isVonNBounded_of_smul_tendsto_zero (by exact hΡ self_mem_nhdsWithin)⟩
235237

0 commit comments

Comments
Β (0)