Monoid actions continuous in the second variable #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
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 #
has_continuous_const_smul Γ T
: typeclass saying that the mapx ↦ γ • x
is continuous onT
;properly_discontinuous_smul
: says that the scalar multiplication(•) : Γ → T → T
is properly discontinuous, that is, for any pair of compact setsK, L
inT
, only finitely manyγ:Γ
moveK
to have nontrivial intersection withL
.homeomorph.smul
: scalar multiplication by an element of a groupΓ
acting onT
is a homeomorphism ofT
.
Main results #
is_open_map_quotient_mk_mul
: The quotient map by a group action is open.t2_space_of_properly_discontinuous_smul_of_t2_space
: The quotient by a discontinuous group action of a locally compact t2 space is t2.
Tags #
Hausdorff, discrete group, properly discontinuous, quotient space
- 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.
Note that both has_continuous_const_smul α α
and has_continuous_const_smul αᵐᵒᵖ α
are
weaker versions of has_continuous_mul α
.
Instances of this typeclass
- has_continuous_smul.has_continuous_const_smul
- is_scalar_tower.has_continuous_const_smul
- smul_comm_class.has_continuous_const_smul
- has_uniform_continuous_const_smul.to_has_continuous_const_smul
- has_isometric_smul.to_has_continuous_const_smul
- has_continuous_const_smul.op
- mul_opposite.has_continuous_const_smul
- order_dual.has_continuous_const_smul
- order_dual.has_continuous_const_smul'
- prod.has_continuous_const_smul
- pi.has_continuous_const_smul
- units.has_continuous_const_smul
- add_monoid.has_continuous_const_smul_nat
- conj_act.units_has_continuous_const_smul
- add_group.has_continuous_const_smul_int
- quotient_group.has_continuous_const_smul
- continuous_linear_map.has_continuous_const_smul
- division_ring.has_continuous_const_smul_rat
- continuous_multilinear_map.has_continuous_const_smul
- matrix.has_continuous_const_smul
- continuous_map.has_continuous_const_smul
- weak_dual.has_continuous_const_smul
- triv_sq_zero_ext.has_continuous_const_smul
- 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.
Note that both has_continuous_const_vadd α α
and has_continuous_const_vadd αᵐᵒᵖ α
are
weaker versions of has_continuous_add α
.
Instances of this typeclass
- has_continuous_vadd.has_continuous_const_vadd
- vadd_assoc_class.has_continuous_const_vadd
- vadd_comm_class.has_continuous_const_vadd
- has_uniform_continuous_const_vadd.to_has_continuous_const_vadd
- has_isometric_vadd.to_has_continuous_const_vadd
- has_continuous_const_vadd.op
- add_opposite.has_continuous_const_vadd
- order_dual.has_continuous_const_vadd
- order_dual.has_continuous_const_vadd'
- prod.has_continuous_const_vadd
- pi.has_continuous_const_vadd
- add_units.has_continuous_const_vadd
- quotient_add_group.has_continuous_const_vadd
- continuous_map.has_continuous_const_vadd
If a scalar is central, then its right action is continuous when its left action is.
If an additive action is central, then its right action is continuous when its left action is.
The homeomorphism given by affine-addition by an element of an additive group Γ
acting on
T
is a homeomorphism from T
to itself.
Equations
- homeomorph.vadd γ = {to_equiv := add_action.to_perm γ, continuous_to_fun := _, continuous_inv_fun := _}
The homeomorphism given by scalar multiplication by a given element of a group Γ
acting on
T
is a homeomorphism from T
to itself.
Equations
- homeomorph.smul γ = {to_equiv := mul_action.to_perm γ, continuous_to_fun := _, continuous_inv_fun := _}
Scalar multiplication by a non-zero element of a group with zero acting on α
is a
homeomorphism from α
onto itself.
Equations
- homeomorph.smul_of_ne_zero c hc = homeomorph.smul (units.mk0 c hc)
smul
is a closed map in the second argument.
The lemma that smul
is a closed map in the first argument (for a normed space over a complete
normed field) is is_closed_map_smul_left
in analysis.normed_space.finite_dimension
.
smul
is a closed map in the second argument.
The lemma that smul
is a closed map in the first argument (for a normed space over a complete
normed field) is is_closed_map_smul_left
in analysis.normed_space.finite_dimension
.
- finite_disjoint_inter_image : ∀ {K L : set T}, is_compact K → is_compact L → {γ : Γ | has_smul.smul γ '' K ∩ L ≠ ∅}.finite
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 of this typeclass
- finite_disjoint_inter_image : ∀ {K L : set T}, is_compact K → is_compact L → {γ : Γ | has_vadd.vadd γ '' K ∩ L ≠ ∅}.finite
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 of this typeclass
A finite group action is always properly discontinuous.
A finite group action is always properly discontinuous.
The quotient map by a group action is open, i.e. the quotient by a group action is an open quotient.
The quotient map by a group action is open, i.e. the quotient by a group action is an open quotient.
The quotient by a discontinuous group action of a locally compact t2 space is t2.
The quotient by a discontinuous group action of a locally compact t2 space is t2.
The quotient of a second countable space by an additive group action is second countable.
The quotient of a second countable space by a group action is second countable.
Scalar multiplication preserves neighborhoods.