Skip to content

Commit aa53d9b

Browse files
committed
chore(Analysis/LocallyConvex): rename a boundedness lemma (#31620)
It was requested in #30523 that the corresponding lemma for `IsCompact` should be called `sUnion_isCompact_eq_univ`, so this one should be `sUnion_isVonNBounded_eq_univ`.
1 parent a3b56a9 commit aa53d9b

File tree

3 files changed

+9
-6
lines changed

3 files changed

+9
-6
lines changed

Mathlib/Analysis/LocallyConvex/Bounded.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -343,10 +343,13 @@ theorem isVonNBounded_sub :
343343
end IsTopologicalAddGroup
344344

345345
/-- The union of all bounded set is the whole space. -/
346-
theorem isVonNBounded_covers : ⋃₀ setOf (IsVonNBounded 𝕜) = (Set.univ : Set E) :=
346+
theorem sUnion_isVonNBounded_eq_univ : ⋃₀ setOf (IsVonNBounded 𝕜) = (Set.univ : Set E) :=
347347
Set.eq_univ_iff_forall.mpr fun x =>
348348
Set.mem_sUnion.mpr ⟨{x}, isVonNBounded_singleton _, Set.mem_singleton _⟩
349349

350+
@[deprecated (since := "2025-11-14")]
351+
alias isVonNBounded_covers := sUnion_isVonNBounded_eq_univ
352+
350353
variable (𝕜 E)
351354

352355
-- See note [reducible non-instances]

Mathlib/Topology/Algebra/Module/Multilinear/Topology.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -83,7 +83,7 @@ lemma isEmbedding_toUniformOnFun :
8383

8484
theorem uniformContinuous_coe_fun [∀ i, ContinuousSMul 𝕜 (E i)] :
8585
UniformContinuous (DFunLike.coe : ContinuousMultilinearMap 𝕜 E F → (Π i, E i) → F) :=
86-
(UniformOnFun.uniformContinuous_toFun isVonNBounded_covers).comp
86+
(UniformOnFun.uniformContinuous_toFun sUnion_isVonNBounded_eq_univ).comp
8787
isUniformEmbedding_toUniformOnFun.uniformContinuous
8888

8989
theorem uniformContinuous_eval_const [∀ i, ContinuousSMul 𝕜 (E i)] (x : Π i, E i) :
@@ -126,7 +126,7 @@ theorem completeSpace (h : IsCoherentWith {s : Set (Π i, E i) | IsVonNBounded
126126
simp [DFunLike.ext_iff]
127127
have H : ∀ {m : Π i, E i},
128128
Continuous fun f : (Π i, E i) →ᵤ[{s | IsVonNBounded 𝕜 s}] F ↦ toFun _ f m :=
129-
(uniformContinuous_eval (isVonNBounded_covers) _).continuous
129+
(uniformContinuous_eval (sUnion_isVonNBounded_eq_univ) _).continuous
130130
rw [completeSpace_iff_isComplete_range isUniformInducing_toUniformOnFun, range_toUniformOnFun]
131131
simp only [setOf_and, setOf_forall]
132132
apply_rules [IsClosed.isComplete, IsClosed.inter]

Mathlib/Topology/Algebra/Module/StrongTopology.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -366,11 +366,11 @@ instance isUniformAddGroup [UniformSpace F] [IsUniformAddGroup F] :
366366

367367
instance instContinuousEvalConst [TopologicalSpace F] [IsTopologicalAddGroup F]
368368
[ContinuousSMul 𝕜₁ E] : ContinuousEvalConst (E →SL[σ] F) E F :=
369-
UniformConvergenceCLM.continuousEvalConst σ F _ Bornology.isVonNBounded_covers
369+
UniformConvergenceCLM.continuousEvalConst σ F _ Bornology.sUnion_isVonNBounded_eq_univ
370370

371371
instance instT2Space [TopologicalSpace F] [IsTopologicalAddGroup F] [ContinuousSMul 𝕜₁ E]
372372
[T2Space F] : T2Space (E →SL[σ] F) :=
373-
UniformConvergenceCLM.t2Space σ F _ Bornology.isVonNBounded_covers
373+
UniformConvergenceCLM.t2Space σ F _ Bornology.sUnion_isVonNBounded_eq_univ
374374

375375
protected theorem hasBasis_nhds_zero_of_basis [TopologicalSpace F] [IsTopologicalAddGroup F]
376376
{ι : Type*} {p : ι → Prop} {b : ι → Set F} (h : (𝓝 0 : Filter F).HasBasis p b) :
@@ -450,7 +450,7 @@ theorem isVonNBounded_iff {R : Type*} [NormedDivisionRing R]
450450
theorem completeSpace [UniformSpace F] [IsUniformAddGroup F] [ContinuousSMul 𝕜₂ F] [CompleteSpace F]
451451
[ContinuousSMul 𝕜₁ E] (h : IsCoherentWith {s : Set E | IsVonNBounded 𝕜₁ s}) :
452452
CompleteSpace (E →SL[σ] F) :=
453-
UniformConvergenceCLM.completeSpace _ _ h isVonNBounded_covers
453+
UniformConvergenceCLM.completeSpace _ _ h sUnion_isVonNBounded_eq_univ
454454

455455
instance instCompleteSpace [IsTopologicalAddGroup E] [ContinuousSMul 𝕜₁ E] [SequentialSpace E]
456456
[UniformSpace F] [IsUniformAddGroup F] [ContinuousSMul 𝕜₂ F] [CompleteSpace F] :

0 commit comments

Comments
 (0)