mathlib3 documentation

topology.algebra.continuous_monoid_hom

Continuous Monoid Homs #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines the space of continuous homomorphisms between two topological groups.

Main definitions #

structure continuous_add_monoid_hom (A : Type u_7) (B : Type u_8) [add_monoid A] [add_monoid B] [topological_space A] [topological_space B] :
Type (max u_7 u_8)

The type of continuous additive monoid homomorphisms from A to B.

When possible, instead of parametrizing results over (f : continuous_add_monoid_hom A B), you should parametrize over (F : Type*) [continuous_add_monoid_hom_class F A B] (f : F).

When you extend this structure, make sure to extend continuous_add_monoid_hom_class.

Instances for continuous_add_monoid_hom
structure continuous_monoid_hom (A : Type u_2) (B : Type u_3) [monoid A] [monoid B] [topological_space A] [topological_space B] :
Type (max u_2 u_3)

The type of continuous monoid homomorphisms from A to B.

When possible, instead of parametrizing results over (f : continuous_monoid_hom A B), you should parametrize over (F : Type*) [continuous_monoid_hom_class F A B] (f : F).

When you extend this structure, make sure to extend continuous_add_monoid_hom_class.

Instances for continuous_monoid_hom
@[class]
structure continuous_add_monoid_hom_class (F : Type u_1) (A : Type u_7) (B : Type u_8) [add_monoid A] [add_monoid B] [topological_space A] [topological_space B] :
Type (max u_1 u_7 u_8)

continuous_add_monoid_hom_class F A B states that F is a type of continuous additive monoid homomorphisms.

You should also extend this typeclass when you extend continuous_add_monoid_hom.

Instances of this typeclass
Instances of other typeclasses for continuous_add_monoid_hom_class
  • continuous_add_monoid_hom_class.has_sizeof_inst
@[class]
structure continuous_monoid_hom_class (F : Type u_1) (A : Type u_2) (B : Type u_3) [monoid A] [monoid B] [topological_space A] [topological_space B] :
Type (max u_1 u_2 u_3)

continuous_monoid_hom_class F A B states that F is a type of continuous additive monoid homomorphisms.

You should also extend this typeclass when you extend continuous_monoid_hom.

Instances of this typeclass
Instances of other typeclasses for continuous_monoid_hom_class
  • continuous_monoid_hom_class.has_sizeof_inst
@[protected, instance]

Helper instance for when there's too many metavariables to apply fun_like.has_coe_to_fun directly.

Equations
@[protected, instance]

Helper instance for when there's too many metavariables to apply fun_like.has_coe_to_fun directly.

Equations
theorem continuous_add_monoid_hom.ext {A : Type u_2} {B : Type u_3} [add_monoid A] [add_monoid B] [topological_space A] [topological_space B] {f g : continuous_add_monoid_hom A B} (h : (x : A), f x = g x) :
f = g
@[ext]
theorem continuous_monoid_hom.ext {A : Type u_2} {B : Type u_3} [monoid A] [monoid B] [topological_space A] [topological_space B] {f g : continuous_monoid_hom A B} (h : (x : A), f x = g x) :
f = g
@[simp]

Composition of two continuous homomorphisms.

Equations

Product of two continuous homomorphisms on the same space.

Equations

Product of two continuous homomorphisms on the same space.

Equations

Product of two continuous homomorphisms on different spaces.

Equations

Product of two continuous homomorphisms on different spaces.

Equations

The trivial continuous homomorphism.

Equations

The continuous homomorphism given by projection onto the first factor.

Equations

The continuous homomorphism given by projection onto the first factor.

Equations

The continuous homomorphism given by projection onto the second factor.

Equations

The continuous homomorphism given by projection onto the second factor.

Equations

The continuous homomorphism given by inclusion of the first factor.

Equations

The continuous homomorphism given by inclusion of the first factor.

Equations

The continuous homomorphism given by inclusion of the second factor.

Equations

The continuous homomorphism given by inclusion of the second factor.

Equations

The continuous homomorphism given by the diagonal embedding.

Equations

The continuous homomorphism given by the diagonal embedding.

Equations

The continuous homomorphism given by swapping components.

Equations

The continuous homomorphism given by swapping components.

Equations

The continuous homomorphism given by multiplication.

Equations

Coproduct of two continuous homomorphisms to the same space.

Equations

Coproduct of two continuous homomorphisms to the same space.

Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
@[protected, instance]
@[protected, instance]
@[protected, instance]
@[protected, instance]
@[simp]
theorem pontryagin_dual.map_apply {A : Type u_2} {B : Type u_3} [monoid A] [monoid B] [topological_space A] [topological_space B] (f : continuous_monoid_hom A B) (x : pontryagin_dual B) (y : A) :