mathlib documentation

topology.algebra.const_mul_action

Monoid actions continuous in the second variable #

In this file we define class has_continuous_const_smul. We say has_continuous_const_smul Γ T if Γ acts on T and for each γ, the map x ↦ γ • x is continuous. (This differs from has_continuous_smul, which requires simultaneous continuity in both variables.)

Main definitions #

Main results #

Tags #

Hausdorff, discrete group, properly discontinuous, quotient space

@[class]
structure has_continuous_const_smul (Γ : Type u_1) (T : Type u_2) [topological_space T] [has_scalar Γ T] :
Prop
  • continuous_const_smul : ∀ (γ : Γ), continuous (λ (x : T), γ x)

Class has_continuous_const_smul Γ T says that the scalar multiplication (•) : Γ → T → T is continuous in the second argument. We use the same class for all kinds of multiplicative actions, including (semi)modules and algebras.

Instances
@[class]
structure has_continuous_const_vadd (Γ : Type u_1) (T : Type u_2) [topological_space T] [has_vadd Γ T] :
Prop
  • continuous_const_vadd : ∀ (γ : Γ), continuous (λ (x : T), γ +ᵥ x)

Class has_continuous_const_vadd Γ T says that the additive action (+ᵥ) : Γ → T → T is continuous in the second argument. We use the same class for all kinds of additive actions, including (semi)modules and algebras.

Instances
@[class]
structure properly_discontinuous_smul (Γ : Type u_1) (T : Type u_2) [topological_space T] [has_scalar Γ T] :
Prop

Class properly_discontinuous_smul Γ T says that the scalar multiplication (•) : Γ → T → T is properly discontinuous, that is, for any pair of compact sets K, L in T, only finitely many γ:Γ move K to have nontrivial intersection with L.

Instances
@[class]
structure properly_discontinuous_vadd (Γ : Type u_1) (T : Type u_2) [topological_space T] [has_vadd Γ T] :
Prop

Class properly_discontinuous_vadd Γ T says that the additive action (+ᵥ) : Γ → T → T is properly discontinuous, that is, for any pair of compact sets K, L in T, only finitely many γ:Γ move K to have nontrivial intersection with L.

Instances
@[protected, instance]
def fintype.properly_discontinuous_vadd {Γ : Type u_1} [add_group Γ] {T : Type u_2} [topological_space T] [add_action Γ T] [fintype Γ] :
@[protected, instance]
def fintype.properly_discontinuous_smul {Γ : Type u_1} [group Γ] {T : Type u_2} [topological_space T] [mul_action Γ T] [fintype Γ] :

A finite group action is always properly discontinuous

def homeomorph.smul {T : Type u_1} [topological_space T] {Γ : Type u_2} [group Γ] [mul_action Γ T] [has_continuous_const_smul Γ T] (γ : Γ) :
T ≃ₜ T

The homeomorphism given by scalar multiplication by a given element of a group Γ acting on T is a homeomorphism from T to itself.

Equations
def homeomorph.vadd {T : Type u_1} [topological_space T] {Γ : Type u_2} [add_group Γ] [add_action Γ T] [has_continuous_const_vadd Γ T] (γ : Γ) :
T ≃ₜ T

The homeomorphism given by affine-addition by an element of an additive group Γ acting on T is a homeomorphism from T to itself.

Equations
theorem is_open_map_quotient_mk_mul {Γ : Type u_1} [group Γ] {T : Type u_2} [topological_space T] [mul_action Γ T] [has_continuous_const_smul Γ T] :

The quotient map by a group action is open.

@[protected, instance]

The quotient by a discontinuous group action of a locally compact t2 space is t2.