Documentation

Mathlib.Topology.Algebra.NonUnitalStarAlgebra

Non-unital topological star (sub)algebras #

A non-unital topological star algebra over a topological semiring R is a topological (non-unital) semiring with a compatible continuous scalar multiplication by elements of R and a continuous star operation. We reuse typeclasses ContinuousSMul and ContinuousStar to express the latter two conditions.

Results #

Any non-unital star subalgebra of a non-unital topological star algebra is itself a non-unital topological star algebra, and its closure is again a non-unital star subalgebra.

The (topological) closure of a non-unital star subalgebra of a non-unital topological star algebra is itself a non-unital star subalgebra.

Equations
  • s.topologicalClosure = { carrier := closure s, add_mem' := , zero_mem' := , mul_mem' := , smul_mem' := , star_mem' := }
Instances For
    @[reducible, inline]

    If a non-unital star subalgebra of a non-unital topological star algebra is commutative, then so is its topological closure.

    See note [reducible non-instances]

    Equations
    • s.nonUnitalCommSemiringTopologicalClosure hs = s.nonUnitalCommSemiringTopologicalClosure hs
    Instances For
      @[reducible, inline]
      abbrev NonUnitalStarSubalgebra.nonUnitalCommRingTopologicalClosure {R : Type u_1} {A : Type u_2} [CommRing R] [TopologicalSpace A] [NonUnitalRing A] [Module R A] [Star A] [TopologicalRing A] [ContinuousStar A] [ContinuousConstSMul R A] [T2Space A] (s : NonUnitalStarSubalgebra R A) (hs : ∀ (x y : s), x * y = y * x) :
      NonUnitalCommRing s.topologicalClosure

      If a non-unital star subalgebra of a non-unital topological star algebra is commutative, then so is its topological closure.

      See note [reducible non-instances].

      Equations
      Instances For