Documentation

Mathlib.Topology.Algebra.SeparationQuotient.Hom

Lift of MonoidHom M N to MonoidHom (SeparationQuotient M) N #

In this file we define the lift of a continuous monoid homomorphism f from M to N to SeparationQuotient M, assuming that f maps two inseparable elements to the same element.

noncomputable def SeparationQuotient.liftContinuousMonoidHom {M : Type u_1} {N : Type u_2} [TopologicalSpace M] [TopologicalSpace N] [CommMonoid M] [ContinuousMul M] [CommMonoid N] (f : ContinuousMonoidHom M N) (hf : ∀ (x y : M), Inseparable x yf x = f y) :

The lift of a monoid hom from M to a monoid hom from SeparationQuotient M.

Equations
Instances For

    The lift of an additive monoid hom from M to an additive monoid hom from SeparationQuotient M.

    Equations
    Instances For
      @[simp]
      theorem SeparationQuotient.liftContinuousCommMonoidHom_mk {M : Type u_1} {N : Type u_2} [TopologicalSpace M] [TopologicalSpace N] [CommMonoid M] [ContinuousMul M] [CommMonoid N] (f : ContinuousMonoidHom M N) (hf : ∀ (x y : M), Inseparable x yf x = f y) (x : M) :
      @[simp]
      theorem SeparationQuotient.liftContinuousAddCommMonoidHom_mk {M : Type u_1} {N : Type u_2} [TopologicalSpace M] [TopologicalSpace N] [AddCommMonoid M] [ContinuousAdd M] [AddCommMonoid N] (f : ContinuousAddMonoidHom M N) (hf : ∀ (x y : M), Inseparable x yf x = f y) (x : M) :