Commit 2024-04-13 12:00 7a71e528
View on Github →Feat (GroupTheory/GroupAction/Hom/Pointwise) : generalize smul set lemmas to group actions (#12023)
This is a generalization of Mathlib/Algebra/Module/LinearMap/Pointwise.lean
from LinearMapClass
to MulActionHomClass
.
The preexisting lemmas are generalized.
image_smul_setₛₗ
: under aσ
-equivariant map, one hash '' (c • s) = (σ c) • h '' s
.preimage_smul_setₛₗ'
is a general version of the equalityh ⁻¹' (σ c • s) = c • h⁻¹' s
. It requires thatc
acts surjectively andσ c
acts injectively. It is provided with specific versions:preimage_smul_setₛₗ_of_units
requires thatc
andσ c
are unitsMonoidHom.preimage_smul_setₛₗ
requires thatσ
is aMonoidHom
andc
is a unitMonoidHomClass.preimage_smul_setₛₗ
requires thatσ
belongs to aMonoidHomClass
and thatc
is a unitGroup.preimage_smul_setₛₗ
requires that the types ofc
andσ c
are groupsimage_smul_set
,preimage_smul_set
andGroup.preimage_smul_set
are the variants whenσ
is the identity.