Documentation

Mathlib.Topology.Algebra.NonUnitalAlgebra

Non-unital topological (sub)algebras #

A non-unital topological algebra over a topological semiring R is a topological (non-unital) semiring with a compatible continuous scalar multiplication by elements of R. We reuse typeclass ContinuousSMul to express the latter condition.

Results #

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

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

Equations
  • s.topologicalClosure = { carrier := closure s, add_mem' := , zero_mem' := , mul_mem' := , smul_mem' := }
Instances For
    theorem NonUnitalSubalgebra.topologicalClosure_minimal {R : Type u_1} {A : Type u_2} [CommSemiring R] [TopologicalSpace A] [NonUnitalSemiring A] [Module R A] [TopologicalSemiring A] [ContinuousConstSMul R A] (s : NonUnitalSubalgebra R A) {t : NonUnitalSubalgebra R A} (h : s t) (ht : IsClosed t) :
    s.topologicalClosure t
    @[reducible, inline]
    abbrev NonUnitalSubalgebra.nonUnitalCommSemiringTopologicalClosure {R : Type u_1} {A : Type u_2} [CommSemiring R] [TopologicalSpace A] [NonUnitalSemiring A] [Module R A] [TopologicalSemiring A] [ContinuousConstSMul R A] [T2Space A] (s : NonUnitalSubalgebra R A) (hs : ∀ (x y : s), x * y = y * x) :
    NonUnitalCommSemiring s.topologicalClosure

    If a non-unital subalgebra of a non-unital topological 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 NonUnitalSubalgebra.nonUnitalCommRingTopologicalClosure {R : Type u_1} {A : Type u_2} [CommRing R] [TopologicalSpace A] [NonUnitalRing A] [Module R A] [TopologicalRing A] [ContinuousConstSMul R A] [T2Space A] (s : NonUnitalSubalgebra R A) (hs : ∀ (x y : s), x * y = y * x) :
      NonUnitalCommRing s.topologicalClosure

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

      See note [reducible non-instances].

      Equations
      Instances For