Pointwise actions of equivariant maps #
image_smul_setₛₗ
: under aσ
-equivariant map, one hasf '' (c • s) = (σ c) • f '' s
.preimage_smul_setₛₗ'
is a general version of the equalityf ⁻¹' (σ c • s) = c • f⁻¹' s
. It requires thatc
acts surjectively andσ c
acts injectively and is provided with specific versions:preimage_smul_setₛₗ_of_isUnit_isUnit
whenc
andσ c
are unitsIsUnit.preimage_smul_setₛₗ
whenσ
belongs to aMonoidHomClass
andc
is a unitMonoidHom.preimage_smul_setₛₗ
whenσ
is aMonoidHom
andc
is a unitGroup.preimage_smul_setₛₗ
: when the types ofc
andσ c
are groups.
image_smul_set
,preimage_smul_set
andGroup.preimage_smul_set
are the variants whenσ
is the identity.
Alias of vadd_preimage_set_subsetₛₗ
.
Alias of smul_preimage_set_subsetₛₗ
.
Translation of preimage is contained in preimage of translation
General version of preimage_smul_setₛₗ
.
This version assumes that the scalar multiplication by c
is surjective
while the scalar multiplication by σ c
is injective.
General version of preimage_vadd_setₛₗ
.
This version assumes that the vector addition of c
is surjective
while the vector addition of σ c
is injective.
preimage_smul_setₛₗ
when both scalars act by unit
Alias of preimage_smul_setₛₗ_of_isUnit_isUnit
.
preimage_smul_setₛₗ
when both scalars act by unit
preimage_smul_setₛₗ
when c
is a unit and σ
is a monoid homomorphism.
Alias of IsAddUnit.preimage_vadd_setₛₗ
.
Alias of IsUnit.preimage_smul_setₛₗ
.
preimage_smul_setₛₗ
when c
is a unit and σ
is a monoid homomorphism.
preimage_smul_setₛₗ
when c
is a unit and σ
is a monoid homomorphism.
preimage_smul_setₛₗ
in the context of groups
Alias of vadd_preimage_set_subset
.
Alias of smul_preimage_set_subset
.
Alias of IsAddUnit.preimage_vadd_set
.
Alias of IsUnit.preimage_smul_set
.