Documentation

Mathlib.Topology.ContinuousFunction.LocallyConstant

The algebra morphism from locally constant functions to continuous functions. #

The inclusion of locally-constant functions into continuous functions as an additive monoid hom.

Instances For
    theorem LocallyConstant.toContinuousMapAddMonoidHom.proof_2 {X : Type u_2} {Y : Type u_1} [TopologicalSpace X] [TopologicalSpace Y] [AddMonoid Y] [ContinuousAdd Y] (x : LocallyConstant X Y) (y : LocallyConstant X Y) :
    ZeroHom.toFun { toFun := LocallyConstant.toContinuousMap, map_zero' := (_ : 0 = 0) } (x + y) = ZeroHom.toFun { toFun := LocallyConstant.toContinuousMap, map_zero' := (_ : 0 = 0) } x + ZeroHom.toFun { toFun := LocallyConstant.toContinuousMap, map_zero' := (_ : 0 = 0) } y
    @[simp]
    theorem LocallyConstant.toContinuousMapAddMonoidHom_apply {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] [AddMonoid Y] [ContinuousAdd Y] (f : LocallyConstant X Y) :
    LocallyConstant.toContinuousMapAddMonoidHom f = f
    @[simp]
    theorem LocallyConstant.toContinuousMapMonoidHom_apply {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] [Monoid Y] [ContinuousMul Y] (f : LocallyConstant X Y) :
    LocallyConstant.toContinuousMapMonoidHom f = f

    The inclusion of locally-constant functions into continuous functions as a multiplicative monoid hom.

    Instances For

      The inclusion of locally-constant functions into continuous functions as a linear map.

      Instances For

        The inclusion of locally-constant functions into continuous functions as an algebra map.

        Instances For