(Scalar) multiplication and (vector) addition as measurable equivalences #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define the following measurable equivalences:
measurable_equiv.smul
: if a groupG
acts onα
by measurable maps, then each elementc : G
defines a measurable automorphism ofα
;measurable_equiv.vadd
: additive version ofmeasurable_equiv.smul
;measurable_equiv.smul₀
: if a group with zeroG
acts onα
by measurable maps, then each nonzero elementc : G
defines a measurable automorphism ofα
;measurable_equiv.mul_left
: ifG
is a group with measurable multiplication, then left multiplication byg : G
is a measurable automorphism ofG
;measurable_equiv.add_left
: additive version ofmeasurable_equiv.mul_left
;measurable_equiv.mul_right
: ifG
is a group with measurable multiplication, then right multiplication byg : G
is a measurable automorphism ofG
;measurable_equiv.add_right
: additive version ofmeasurable_equiv.mul_right
;measurable_equiv.mul_left₀
,measurable_equiv.mul_right₀
: versions ofmeasurable_equiv.mul_left
andmeasurable_equiv.mul_right
for groups with zero;measurable_equiv.inv
:has_inv.inv
as a measurable automorphism of a group (or a group with zero);measurable_equiv.neg
: negation as a measurable automorphism of an additive group.
We also deduce that the corresponding maps are measurable embeddings.
Tags #
measurable, equivalence, group action
If an additive group G
acts on α
by measurable maps, then each element c : G
defines a measurable automorphism of α
.
Equations
- measurable_equiv.vadd c = {to_equiv := add_action.to_perm c, measurable_to_fun := _, measurable_inv_fun := _}
If a group G
acts on α
by measurable maps, then each element c : G
defines a measurable
automorphism of α
.
Equations
- measurable_equiv.smul c = {to_equiv := mul_action.to_perm c, measurable_to_fun := _, measurable_inv_fun := _}
If a group with zero G₀
acts on α
by measurable maps, then each nonzero element c : G₀
defines a measurable automorphism of α
Equations
- measurable_equiv.smul₀ c hc = measurable_equiv.smul (units.mk0 c hc)
If G
is a group with measurable multiplication, then left multiplication by g : G
is a
measurable automorphism of G
.
Equations
If G
is an additive group with measurable addition, then addition of g : G
on the left is a measurable automorphism of G
.
Equations
If G
is a group with measurable multiplication, then right multiplication by g : G
is a
measurable automorphism of G
.
Equations
- measurable_equiv.mul_right g = {to_equiv := equiv.mul_right g, measurable_to_fun := _, measurable_inv_fun := _}
If G
is an additive group with measurable addition, then addition of g : G
on the right is a measurable automorphism of G
.
Equations
- measurable_equiv.add_right g = {to_equiv := equiv.add_right g, measurable_to_fun := _, measurable_inv_fun := _}
If G₀
is a group with zero with measurable multiplication, then left multiplication by a
nonzero element g : G₀
is a measurable automorphism of G₀
.
Equations
If G₀
is a group with zero with measurable multiplication, then right multiplication by a
nonzero element g : G₀
is a measurable automorphism of G₀
.
Equations
- measurable_equiv.mul_right₀ g hg = {to_equiv := equiv.mul_right₀ g hg, measurable_to_fun := _, measurable_inv_fun := _}
Inversion as a measurable automorphism of a group or group with zero.
Equations
- measurable_equiv.inv G = {to_equiv := equiv.inv G _inst_11, measurable_to_fun := _, measurable_inv_fun := _}
Negation as a measurable automorphism of an additive group.
Equations
- measurable_equiv.neg G = {to_equiv := equiv.neg G _inst_11, measurable_to_fun := _, measurable_inv_fun := _}
equiv.div_right
as a measurable_equiv
.
Equations
- measurable_equiv.div_right g = {to_equiv := equiv.div_right g, measurable_to_fun := _, measurable_inv_fun := _}
equiv.sub_right
as a measurable_equiv
Equations
- measurable_equiv.sub_right g = {to_equiv := equiv.sub_right g, measurable_to_fun := _, measurable_inv_fun := _}
equiv.div_left
as a measurable_equiv
Equations
- measurable_equiv.div_left g = {to_equiv := equiv.div_left g, measurable_to_fun := _, measurable_inv_fun := _}
equiv.sub_left
as a measurable_equiv
Equations
- measurable_equiv.sub_left g = {to_equiv := equiv.sub_left g, measurable_to_fun := _, measurable_inv_fun := _}