Documentation

Mathlib.Analysis.LocallyConvex.AbsConvex

Absolutely convex sets #

A set is called absolutely convex or disked if it is convex and balanced. The importance of absolutely convex sets comes from the fact that every locally convex topological vector space has a basis consisting of absolutely convex sets.

Main definitions #

Main statements #

Todo #

Tags #

disks, convex, balanced

theorem nhds_basis_abs_convex (𝕜 : Type u_1) (E : Type u_2) [NontriviallyNormedField 𝕜] [AddCommGroup E] [Module 𝕜 E] [Module E] [SMulCommClass 𝕜 E] [TopologicalSpace E] [LocallyConvexSpace E] [ContinuousSMul 𝕜 E] :
Filter.HasBasis (nhds 0) (fun (s : Set E) => s nhds 0 Balanced 𝕜 s Convex s) id
def AbsConvexOpenSets (𝕜 : Type u_1) (E : Type u_2) [TopologicalSpace E] [AddCommMonoid E] [Zero E] [SeminormedRing 𝕜] [SMul 𝕜 E] [SMul E] :
Type u_2

The type of absolutely convex open sets.

Equations
Instances For
    noncomputable instance AbsConvexOpenSets.instCoeTC (𝕜 : Type u_1) (E : Type u_2) [TopologicalSpace E] [AddCommMonoid E] [Zero E] [SeminormedRing 𝕜] [SMul 𝕜 E] [SMul E] :
    Equations
    theorem AbsConvexOpenSets.coe_zero_mem {𝕜 : Type u_1} {E : Type u_2} [TopologicalSpace E] [AddCommMonoid E] [Zero E] [SeminormedRing 𝕜] [SMul 𝕜 E] [SMul E] (s : AbsConvexOpenSets 𝕜 E) :
    0 s
    theorem AbsConvexOpenSets.coe_isOpen {𝕜 : Type u_1} {E : Type u_2} [TopologicalSpace E] [AddCommMonoid E] [Zero E] [SeminormedRing 𝕜] [SMul 𝕜 E] [SMul E] (s : AbsConvexOpenSets 𝕜 E) :
    IsOpen s
    theorem AbsConvexOpenSets.coe_nhds {𝕜 : Type u_1} {E : Type u_2} [TopologicalSpace E] [AddCommMonoid E] [Zero E] [SeminormedRing 𝕜] [SMul 𝕜 E] [SMul E] (s : AbsConvexOpenSets 𝕜 E) :
    s nhds 0
    theorem AbsConvexOpenSets.coe_balanced {𝕜 : Type u_1} {E : Type u_2} [TopologicalSpace E] [AddCommMonoid E] [Zero E] [SeminormedRing 𝕜] [SMul 𝕜 E] [SMul E] (s : AbsConvexOpenSets 𝕜 E) :
    Balanced 𝕜 s
    theorem AbsConvexOpenSets.coe_convex {𝕜 : Type u_1} {E : Type u_2} [TopologicalSpace E] [AddCommMonoid E] [Zero E] [SeminormedRing 𝕜] [SMul 𝕜 E] [SMul E] (s : AbsConvexOpenSets 𝕜 E) :
    Convex s
    instance AbsConvexOpenSets.instNonempty (𝕜 : Type u_1) (E : Type u_2) [TopologicalSpace E] [AddCommMonoid E] [Zero E] [SeminormedRing 𝕜] [SMul 𝕜 E] [SMul E] :
    Equations
    • =
    noncomputable def gaugeSeminormFamily (𝕜 : Type u_1) (E : Type u_2) [RCLike 𝕜] [AddCommGroup E] [TopologicalSpace E] [Module 𝕜 E] [Module E] [IsScalarTower 𝕜 E] [ContinuousSMul E] :

    The family of seminorms defined by the gauges of absolute convex open sets.

    Equations
    Instances For
      theorem gaugeSeminormFamily_ball {𝕜 : Type u_1} {E : Type u_2} [RCLike 𝕜] [AddCommGroup E] [TopologicalSpace E] [Module 𝕜 E] [Module E] [IsScalarTower 𝕜 E] [ContinuousSMul E] (s : AbsConvexOpenSets 𝕜 E) :
      Seminorm.ball (gaugeSeminormFamily 𝕜 E s) 0 1 = s

      The topology of a locally convex space is induced by the gauge seminorm family.