Sets invariant to a mul_action #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define sub_mul_action R M; a subset of a mul_action R M which is closed with
respect to scalar multiplication.
For most uses, typically submodule R M is more powerful.
Main definitions #
- sub_mul_action.mul_action- the- mul_action R Mtransferred to the subtype.
- sub_mul_action.mul_action'- the- mul_action S Mtransferred to the subtype when- is_scalar_tower S R M.
- sub_mul_action.is_scalar_tower- the- is_scalar_tower S R Mtransferred to the subtype.
Tags #
submodule, mul_action
smul_mem_class S R M says S is a type of subsets s ≤ M that are closed under the
scalar action of R on M.
Note that only R is marked as an out_param here, since M is supplied by the set_like
class instead.
Instances of this typeclass
Instances of other typeclasses for smul_mem_class
        
        - smul_mem_class.has_sizeof_inst
vadd_mem_class S R M says S is a type of subsets s ≤ M that are closed under the
additive action of R on M.
Note that only R is marked as an out_param here, since M is supplied by the set_like
class instead.
Instances for vadd_mem_class
        
        - vadd_mem_class.has_sizeof_inst
A subset closed under the additive action inherits that action.
A subset closed under the scalar action inherits that action.
A sub_mul_action is a set which is closed under scalar multiplication.
Instances for sub_mul_action
        
        
    Equations
- sub_mul_action.set_like = {coe := sub_mul_action.carrier _inst_1, coe_injective' := _}
Equations
Copy of a sub_mul_action with a new carrier equal to the old one. Useful to fix definitional
equalities.
Equations
A sub_mul_action of a mul_action is a mul_action.
Equations
The natural mul_action_hom over R from a sub_mul_action of M to M.
Equations
- sub_mul_action.smul_mem_class.subtype S' = {to_fun := coe coe_to_lift, map_smul' := _}
If the scalar product forms a mul_action, then the subset inherits this action
Equations
- p.mul_action' = {to_has_smul := {smul := has_smul.smul p.has_smul'}, one_smul := _, mul_smul := _}
Equations
- p.mul_action = p.mul_action'
Orbits in a sub_mul_action coincide with orbits in the ambient space.
Stabilizers in monoid sub_mul_action coincide with stabilizers in the ambient space
Stabilizers in group sub_mul_action coincide with stabilizers in the ambient space
If the scalar product forms a module, and the sub_mul_action is not ⊥, then the
subset inherits the zero.