Documentation

Mathlib.Analysis.LocallyConvex.Bounded

Von Neumann Boundedness #

This file defines natural or von Neumann bounded sets and proves elementary properties.

Main declarations #

Main results #

References #

def Bornology.IsVonNBounded (๐•œ : Type u_1) {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] (s : Set E) :

A set s is von Neumann bounded if every neighborhood of 0 absorbs s.

Equations
Instances For
    @[simp]
    theorem Bornology.isVonNBounded_empty (๐•œ : Type u_1) (E : Type u_3) [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] :
    theorem Bornology.isVonNBounded_iff {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] (s : Set E) :
    IsVonNBounded ๐•œ s โ†” โˆ€ V โˆˆ nhds 0, Absorbs ๐•œ V s
    theorem Filter.HasBasis.isVonNBounded_iff {๐•œ : Type u_1} {E : Type u_3} {ฮน : Type u_5} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] {q : ฮน โ†’ Prop} {s : ฮน โ†’ Set E} {A : Set E} (h : (nhds 0).HasBasis q s) :
    Bornology.IsVonNBounded ๐•œ A โ†” โˆ€ (i : ฮน), q i โ†’ Absorbs ๐•œ (s i) A
    theorem Bornology.IsVonNBounded.subset {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] {sโ‚ sโ‚‚ : Set E} (h : sโ‚ โІ sโ‚‚) (hsโ‚‚ : IsVonNBounded ๐•œ sโ‚‚) :
    IsVonNBounded ๐•œ sโ‚

    Subsets of bounded sets are bounded.

    @[simp]
    theorem Bornology.isVonNBounded_union {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] {s t : Set E} :
    IsVonNBounded ๐•œ (s โˆช t) โ†” IsVonNBounded ๐•œ s โˆง IsVonNBounded ๐•œ t
    theorem Bornology.IsVonNBounded.union {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] {sโ‚ sโ‚‚ : Set E} (hsโ‚ : IsVonNBounded ๐•œ sโ‚) (hsโ‚‚ : IsVonNBounded ๐•œ sโ‚‚) :
    IsVonNBounded ๐•œ (sโ‚ โˆช sโ‚‚)

    The union of two bounded sets is bounded.

    theorem Bornology.IsVonNBounded.of_boundedSpace {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] [BoundedSpace ๐•œ] {s : Set E} :
    IsVonNBounded ๐•œ s
    theorem Bornology.IsVonNBounded.of_subsingleton {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] [Subsingleton E] {s : Set E} :
    IsVonNBounded ๐•œ s
    @[simp]
    theorem Bornology.isVonNBounded_iUnion {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] {ฮน : Sort u_6} [Finite ฮน] {s : ฮน โ†’ Set E} :
    IsVonNBounded ๐•œ (โ‹ƒ (i : ฮน), s i) โ†” โˆ€ (i : ฮน), IsVonNBounded ๐•œ (s i)
    theorem Bornology.isVonNBounded_biUnion {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] {ฮน : Type u_6} {I : Set ฮน} (hI : I.Finite) {s : ฮน โ†’ Set E} :
    IsVonNBounded ๐•œ (โ‹ƒ i โˆˆ I, s i) โ†” โˆ€ i โˆˆ I, IsVonNBounded ๐•œ (s i)
    theorem Bornology.isVonNBounded_sUnion {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [SMul ๐•œ E] [Zero E] [TopologicalSpace E] {S : Set (Set E)} (hS : S.Finite) :
    IsVonNBounded ๐•œ (โ‹ƒโ‚€ S) โ†” โˆ€ s โˆˆ S, IsVonNBounded ๐•œ s
    theorem Bornology.IsVonNBounded.add {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [AddZeroClass E] [TopologicalSpace E] [ContinuousAdd E] [DistribSMul ๐•œ E] {s t : Set E} (hs : IsVonNBounded ๐•œ s) (ht : IsVonNBounded ๐•œ t) :
    IsVonNBounded ๐•œ (s + t)
    theorem Bornology.IsVonNBounded.neg {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [AddGroup E] [TopologicalSpace E] [IsTopologicalAddGroup E] [DistribMulAction ๐•œ E] {s : Set E} (hs : IsVonNBounded ๐•œ s) :
    IsVonNBounded ๐•œ (-s)
    @[simp]
    theorem Bornology.isVonNBounded_neg {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [AddGroup E] [TopologicalSpace E] [IsTopologicalAddGroup E] [DistribMulAction ๐•œ E] {s : Set E} :
    IsVonNBounded ๐•œ (-s) โ†” IsVonNBounded ๐•œ s
    theorem Bornology.IsVonNBounded.of_neg {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [AddGroup E] [TopologicalSpace E] [IsTopologicalAddGroup E] [DistribMulAction ๐•œ E] {s : Set E} :
    IsVonNBounded ๐•œ (-s) โ†’ IsVonNBounded ๐•œ s

    Alias of the forward direction of Bornology.isVonNBounded_neg.

    theorem Bornology.IsVonNBounded.sub {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [AddGroup E] [TopologicalSpace E] [IsTopologicalAddGroup E] [DistribMulAction ๐•œ E] {s t : Set E} (hs : IsVonNBounded ๐•œ s) (ht : IsVonNBounded ๐•œ t) :
    IsVonNBounded ๐•œ (s - t)
    theorem Bornology.IsVonNBounded.of_topologicalSpace_le {๐•œ : Type u_1} {E : Type u_3} [SeminormedRing ๐•œ] [AddCommGroup E] [Module ๐•œ E] {t t' : TopologicalSpace E} (h : t โ‰ค t') {s : Set E} (hs : IsVonNBounded ๐•œ s) :
    IsVonNBounded ๐•œ s

    If a topology t' is coarser than t, then any set s that is bounded with respect to t is bounded with respect to t'.

    theorem Bornology.isVonNBounded_iff_tendsto_smallSets_nhds {๐•œ : Type u_6} {E : Type u_7} [NormedDivisionRing ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] {S : Set E} :
    IsVonNBounded ๐•œ S โ†” Filter.Tendsto (fun (x : ๐•œ) => x โ€ข S) (nhds 0) (nhds 0).smallSets
    theorem Bornology.IsVonNBounded.tendsto_smallSets_nhds {๐•œ : Type u_6} {E : Type u_7} [NormedDivisionRing ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] {S : Set E} :
    IsVonNBounded ๐•œ S โ†’ Filter.Tendsto (fun (x : ๐•œ) => x โ€ข S) (nhds 0) (nhds 0).smallSets

    Alias of the forward direction of Bornology.isVonNBounded_iff_tendsto_smallSets_nhds.

    theorem Bornology.isVonNBounded_iff_absorbing_le {๐•œ : Type u_6} {E : Type u_7} [NormedDivisionRing ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] {S : Set E} :
    theorem Bornology.isVonNBounded_pi_iff {๐•œ : Type u_6} {ฮน : Type u_7} {E : ฮน โ†’ Type u_8} [NormedDivisionRing ๐•œ] [(i : ฮน) โ†’ AddCommGroup (E i)] [(i : ฮน) โ†’ Module ๐•œ (E i)] [(i : ฮน) โ†’ TopologicalSpace (E i)] {S : Set ((i : ฮน) โ†’ E i)} :
    IsVonNBounded ๐•œ S โ†” โˆ€ (i : ฮน), IsVonNBounded ๐•œ (Function.eval i '' S)
    theorem Bornology.IsVonNBounded.image {E : Type u_3} {F : Type u_4} {๐•œโ‚ : Type u_6} {๐•œโ‚‚ : Type u_7} [NormedDivisionRing ๐•œโ‚] [NormedDivisionRing ๐•œโ‚‚] [AddCommGroup E] [Module ๐•œโ‚ E] [AddCommGroup F] [Module ๐•œโ‚‚ F] [TopologicalSpace E] [TopologicalSpace F] {ฯƒ : ๐•œโ‚ โ†’+* ๐•œโ‚‚} [RingHomSurjective ฯƒ] [RingHomIsometric ฯƒ] {s : Set E} (hs : IsVonNBounded ๐•œโ‚ s) (f : E โ†’SL[ฯƒ] F) :
    IsVonNBounded ๐•œโ‚‚ (โ‡‘f '' s)

    A continuous linear image of a bounded set is bounded.

    theorem Bornology.IsVonNBounded.smul_tendsto_zero {๐•œ : Type u_1} {E : Type u_3} {ฮน : Type u_5} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] {S : Set E} {ฮต : ฮน โ†’ ๐•œ} {x : ฮน โ†’ E} {l : Filter ฮน} (hS : IsVonNBounded ๐•œ S) (hxS : โˆ€แถ  (n : ฮน) in l, x n โˆˆ S) (hฮต : Filter.Tendsto ฮต l (nhds 0)) :
    Filter.Tendsto (ฮต โ€ข x) l (nhds 0)
    theorem Bornology.isVonNBounded_of_smul_tendsto_zero {๐•œ : Type u_1} {E : Type u_3} {ฮน : Type u_5} [NontriviallyNormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] {ฮต : ฮน โ†’ ๐•œ} {l : Filter ฮน} [l.NeBot] (hฮต : โˆ€แถ  (n : ฮน) in l, ฮต n โ‰  0) {S : Set E} (H : โˆ€ (x : ฮน โ†’ E), (โˆ€ (n : ฮน), x n โˆˆ S) โ†’ Filter.Tendsto (ฮต โ€ข x) l (nhds 0)) :
    IsVonNBounded ๐•œ S
    theorem Bornology.isVonNBounded_iff_smul_tendsto_zero {๐•œ : Type u_1} {E : Type u_3} {ฮน : Type u_5} [NontriviallyNormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] {ฮต : ฮน โ†’ ๐•œ} {l : Filter ฮน} [l.NeBot] (hฮต : Filter.Tendsto ฮต l (nhdsWithin 0 {0}แถœ)) {S : Set E} :
    IsVonNBounded ๐•œ S โ†” โˆ€ (x : ฮน โ†’ E), (โˆ€ (n : ฮน), x n โˆˆ S) โ†’ Filter.Tendsto (ฮต โ€ข x) l (nhds 0)

    Given any sequence ฮต of scalars which tends to ๐“[โ‰ ] 0, we have that a set S is bounded if and only if for any sequence x : โ„• โ†’ S, ฮต โ€ข x tends to 0. This actually works for any indexing type ฮน, but in the special case ฮน = โ„• we get the important fact that convergent sequences fully characterize bounded sets.

    theorem Bornology.IsVonNBounded.extend_scalars {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_6} [AddCommGroup E] [Module ๐•œ E] (๐• : Type u_7) [NontriviallyNormedField ๐•] [NormedAlgebra ๐•œ ๐•] [Module ๐• E] [TopologicalSpace E] [ContinuousSMul ๐• E] [IsScalarTower ๐•œ ๐• E] {s : Set E} (h : IsVonNBounded ๐•œ s) :
    IsVonNBounded ๐• s

    If a set is von Neumann bounded with respect to a smaller field, then it is also von Neumann bounded with respect to a larger field. See also Bornology.IsVonNBounded.restrict_scalars below.

    theorem Bornology.isVonNBounded_singleton {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] (x : E) :
    IsVonNBounded ๐•œ {x}

    Singletons are bounded.

    @[simp]
    theorem Bornology.isVonNBounded_insert {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] (x : E) {s : Set E} :
    IsVonNBounded ๐•œ (insert x s) โ†” IsVonNBounded ๐•œ s
    theorem Bornology.IsVonNBounded.insert {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] (x : E) {s : Set E} :
    IsVonNBounded ๐•œ s โ†’ IsVonNBounded ๐•œ (insert x s)

    Alias of the reverse direction of Bornology.isVonNBounded_insert.

    theorem Bornology.IsVonNBounded.vadd {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [ContinuousAdd E] {s : Set E} (hs : IsVonNBounded ๐•œ s) (x : E) :
    IsVonNBounded ๐•œ (x +แตฅ s)
    @[simp]
    theorem Bornology.isVonNBounded_vadd {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [ContinuousAdd E] {s : Set E} (x : E) :
    IsVonNBounded ๐•œ (x +แตฅ s) โ†” IsVonNBounded ๐•œ s
    theorem Bornology.IsVonNBounded.of_add_right {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [ContinuousAdd E] {s t : Set E} (hst : IsVonNBounded ๐•œ (s + t)) (hs : s.Nonempty) :
    IsVonNBounded ๐•œ t
    theorem Bornology.IsVonNBounded.of_add_left {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [ContinuousAdd E] {s t : Set E} (hst : IsVonNBounded ๐•œ (s + t)) (ht : t.Nonempty) :
    IsVonNBounded ๐•œ s
    theorem Bornology.isVonNBounded_add_of_nonempty {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [ContinuousAdd E] {s t : Set E} (hs : s.Nonempty) (ht : t.Nonempty) :
    IsVonNBounded ๐•œ (s + t) โ†” IsVonNBounded ๐•œ s โˆง IsVonNBounded ๐•œ t
    theorem Bornology.isVonNBounded_add {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [ContinuousAdd E] {s t : Set E} :
    @[simp]
    theorem Bornology.isVonNBounded_add_self {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [ContinuousAdd E] {s : Set E} :
    IsVonNBounded ๐•œ (s + s) โ†” IsVonNBounded ๐•œ s
    theorem Bornology.IsVonNBounded.of_sub_left {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [ContinuousAdd E] {s t : Set E} (hst : IsVonNBounded ๐•œ (s - t)) (ht : t.Nonempty) :
    IsVonNBounded ๐•œ s
    theorem Bornology.IsVonNBounded.of_sub_right {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [IsTopologicalAddGroup E] {s t : Set E} (hst : IsVonNBounded ๐•œ (s - t)) (hs : s.Nonempty) :
    IsVonNBounded ๐•œ t
    theorem Bornology.isVonNBounded_sub_of_nonempty {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [IsTopologicalAddGroup E] {s t : Set E} (hs : s.Nonempty) (ht : t.Nonempty) :
    IsVonNBounded ๐•œ (s - t) โ†” IsVonNBounded ๐•œ s โˆง IsVonNBounded ๐•œ t
    theorem Bornology.isVonNBounded_sub {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] [IsTopologicalAddGroup E] {s t : Set E} :
    theorem Bornology.isVonNBounded_covers {๐•œ : Type u_1} {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] :

    The union of all bounded set is the whole space.

    @[reducible, inline]
    abbrev Bornology.vonNBornology (๐•œ : Type u_1) (E : Type u_3) [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] :

    The von Neumann bornology defined by the von Neumann bounded sets.

    Note that this is not registered as an instance, in order to avoid diamonds with the metric bornology.

    Equations
    Instances For
      @[simp]
      theorem Bornology.isBounded_iff_isVonNBounded (๐•œ : Type u_1) {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [ContinuousSMul ๐•œ E] {s : Set E} :
      theorem TotallyBounded.isVonNBounded (๐•œ : Type u_1) {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [UniformSpace E] [IsUniformAddGroup E] [ContinuousSMul ๐•œ E] {s : Set E} (hs : TotallyBounded s) :
      theorem Filter.Tendsto.isVonNBounded_range (๐•œ : Type u_1) {E : Type u_3} [NormedField ๐•œ] [AddCommGroup E] [Module ๐•œ E] [TopologicalSpace E] [IsTopologicalAddGroup E] [ContinuousSMul ๐•œ E] {f : โ„• โ†’ E} {x : E} (hf : Tendsto f atTop (nhds x)) :
      theorem Bornology.IsVonNBounded.restrict_scalars_of_nontrivial (๐•œ : Type u_1) {๐•œ' : Type u_2} {E : Type u_3} [NormedField ๐•œ] [NormedRing ๐•œ'] [NormedAlgebra ๐•œ ๐•œ'] [Nontrivial ๐•œ'] [Zero E] [TopologicalSpace E] [SMul ๐•œ E] [MulAction ๐•œ' E] [IsScalarTower ๐•œ ๐•œ' E] {s : Set E} (h : IsVonNBounded ๐•œ' s) :
      IsVonNBounded ๐•œ s
      theorem Bornology.IsVonNBounded.restrict_scalars (๐•œ : Type u_1) {๐•œ' : Type u_2} {E : Type u_3} [NormedField ๐•œ] [NormedRing ๐•œ'] [NormedAlgebra ๐•œ ๐•œ'] [Zero E] [TopologicalSpace E] [SMul ๐•œ E] [MulActionWithZero ๐•œ' E] [IsScalarTower ๐•œ ๐•œ' E] {s : Set E} (h : IsVonNBounded ๐•œ' s) :
      IsVonNBounded ๐•œ s
      theorem NormedSpace.isVonNBounded_of_isBounded (๐•œ : Type u_1) {E : Type u_3} [NormedField ๐•œ] [SeminormedAddCommGroup E] [NormedSpace ๐•œ E] {s : Set E} (h : Bornology.IsBounded s) :
      theorem NormedSpace.isVonNBounded_ball (๐•œ : Type u_1) (E : Type u_3) [NormedField ๐•œ] [SeminormedAddCommGroup E] [NormedSpace ๐•œ E] (r : โ„) :
      theorem NormedSpace.isVonNBounded_closedBall (๐•œ : Type u_1) (E : Type u_3) [NormedField ๐•œ] [SeminormedAddCommGroup E] [NormedSpace ๐•œ E] (r : โ„) :
      theorem NormedSpace.isVonNBounded_iff' (๐•œ : Type u_1) {E : Type u_3} [NontriviallyNormedField ๐•œ] [SeminormedAddCommGroup E] [NormedSpace ๐•œ E] {s : Set E} :
      Bornology.IsVonNBounded ๐•œ s โ†” โˆƒ (r : โ„), โˆ€ x โˆˆ s, โ€–xโ€– โ‰ค r
      theorem NormedSpace.image_isVonNBounded_iff (๐•œ : Type u_1) {E : Type u_3} [NontriviallyNormedField ๐•œ] [SeminormedAddCommGroup E] [NormedSpace ๐•œ E] {ฮฑ : Type u_6} {f : ฮฑ โ†’ E} {s : Set ฮฑ} :
      Bornology.IsVonNBounded ๐•œ (f '' s) โ†” โˆƒ (r : โ„), โˆ€ x โˆˆ s, โ€–f xโ€– โ‰ค r

      In a normed space, the von Neumann bornology (Bornology.vonNBornology) is equal to the metric bornology.

      theorem NormedSpace.isBounded_iff_subset_smul_ball (๐•œ : Type u_1) {E : Type u_3} [NontriviallyNormedField ๐•œ] [SeminormedAddCommGroup E] [NormedSpace ๐•œ E] {s : Set E} :
      Bornology.IsBounded s โ†” โˆƒ (a : ๐•œ), s โІ a โ€ข Metric.ball 0 1
      theorem NormedSpace.isBounded_iff_subset_smul_closedBall (๐•œ : Type u_1) {E : Type u_3} [NontriviallyNormedField ๐•œ] [SeminormedAddCommGroup E] [NormedSpace ๐•œ E] {s : Set E} :
      Bornology.IsBounded s โ†” โˆƒ (a : ๐•œ), s โІ a โ€ข Metric.closedBall 0 1
      class QuasiCompleteSpace (๐•œ : Type u_6) (E : Type u_7) [Zero E] [UniformSpace E] [SeminormedRing ๐•œ] [SMul ๐•œ E] :

      A locally convex space is quasi-complete if every closed and von Neumann bounded set is complete.

      Instances
        instance instQuasiCompleteSpaceOfCompleteSpace {๐•œ : Type u_6} {E : Type u_7} [Zero E] [UniformSpace E] [SeminormedRing ๐•œ] [SMul ๐•œ E] [CompleteSpace E] :
        QuasiCompleteSpace ๐•œ E

        A complete space is quasi-complete with respect to any scalar ring.