Equations
- quotient_group.group N = {mul := quotient.map₂' has_mul.mul _, mul_assoc := _, one := ↑1, one_mul := _, mul_one := _, inv := λ (a : quotient_group.quotient N), quotient.lift_on' a (λ (a : G), ↑a⁻¹) _, mul_left_inv := _}
The group homomorphism from G
to G/N
.
Equations
The additive group homomorphism from G
to G/N
.
Equations
- quotient_group.comm_group N = {mul := group.mul (quotient_group.group N), mul_assoc := _, one := group.one (quotient_group.group N), one_mul := _, mul_one := _, inv := group.inv (quotient_group.group N), mul_left_inv := _, mul_comm := _}
An add_group
homomorphism φ : G →+ H
with N ⊆ ker(φ)
descends (i.e. lift
s) to a group homomorphism G/N →* H
.
A group homomorphism φ : G →* H
with N ⊆ ker(φ)
descends (i.e. lift
s) to a
group homomorphism G/N →* H
.
Equations
- quotient_group.lift N φ HN = monoid_hom.mk' (λ (q : quotient_group.quotient N), quotient.lift_on' q ⇑φ _) _
An add_group
homomorphism f : G →+ H
induces a map
G/N →+ H/M
if N ⊆ f⁻¹(M)
.
A group homomorphism f : G →* H
induces a map G/N →* H/M
if N ⊆ f⁻¹(M)
.
Equations
- quotient_group.map N M f h = quotient_group.lift N ((quotient_group.mk' M).comp f) _
The induced map from the quotient by the kernel to the codomain.
The induced map from the quotient by the kernel to the codomain.
Equations
The induced map from the quotient by the kernel to the range.
Equations
The induced map from the quotient by the kernel to the range.
The first isomorphism theorem (a definition): the canonical isomorphism between
G/(ker φ)
to range φ
.
The first isomorphism theorem
(a definition): the canonical isomorphism between G/(ker φ)
to range φ
.
The canonical isomorphism
G/(ker φ) ≃+ H
induced by a surjection φ : G →+ H
.
The canonical isomorphism G/(ker φ) ≃* H
induced by a surjection φ : G →* H
.