Double cosets #
This file defines double cosets for two subgroups H K
of a group G
and the quotient of G
by
the double coset relation, i.e. H \ G / K
. We also prove that G
can be written as a disjoint
union of the double cosets and that if one of H
or K
is the trivial group (i.e. ⊥
) then
this is the usual left or right quotient of a group by a subgroup.
Main definitions #
setoid
: The double coset relation defined by two subgroupsH K
ofG
.DoubleCoset.quotient
: The quotient ofG
by the double coset relation, i.e,H \ G / K
.
Alias of DoubleCoset.doubleCoset
.
The double coset as an element of Set α
corresponding to s a t
Equations
Instances For
Alias of DoubleCoset.doubleCoset_eq_image2
.
Alias of DoubleCoset.mem_doubleCoset
.
Alias of DoubleCoset.mem_doubleCoset_self
.
Alias of DoubleCoset.doubleCoset_eq_of_mem
.
Alias of DoubleCoset.eq_of_not_disjoint
.
The setoid defined by the double_coset relation
Equations
- DoubleCoset.setoid H K = Setoid.ker fun (x : G) => DoubleCoset.doubleCoset x H K
Instances For
Alias of DoubleCoset.setoid
.
The setoid defined by the double_coset relation
Equations
Instances For
Quotient of G
by the double coset relation, i.e. H \ G / K
Equations
- DoubleCoset.Quotient H K = Quotient (DoubleCoset.setoid H K)
Instances For
Alias of DoubleCoset.Quotient
.
Quotient of G
by the double coset relation, i.e. H \ G / K
Equations
Instances For
Alias of DoubleCoset.rel_iff
.
Alias of DoubleCoset.bot_rel_eq_leftRel
.
Alias of DoubleCoset.rel_bot_eq_right_group_rel
.
Create a double coset out of an element of H \ G / K
Equations
- DoubleCoset.quotToDoubleCoset H K q = DoubleCoset.doubleCoset (Quotient.out q) ↑H ↑K
Instances For
Alias of DoubleCoset.quotToDoubleCoset
.
Create a double coset out of an element of H \ G / K
Equations
Instances For
Map from G
to H \ G / K
Equations
- DoubleCoset.mk H K a = Quotient.mk'' a
Instances For
Alias of DoubleCoset.mk
.
Map from G
to H \ G / K
Equations
Instances For
Equations
- DoubleCoset.instInhabitedQuotientCoeSubgroup H K = { default := DoubleCoset.mk H K 1 }
Alias of DoubleCoset.eq
.
Alias of DoubleCoset.out_eq'
.
Alias of DoubleCoset.mk_out_eq_mul
.
Alias of DoubleCoset.mk_eq_of_doubleCoset_eq
.
Alias of DoubleCoset.disjoint_out
.
Alias of DoubleCoset.union_quotToDoubleCoset
.
Alias of DoubleCoset.doubleCoset_union_rightCoset
.
Alias of DoubleCoset.doubleCoset_union_leftCoset
.
Alias of DoubleCoset.left_bot_eq_left_quot
.
Alias of DoubleCoset.right_bot_eq_right_quot
.