Documentation

Mathlib.Algebra.Category.Grp.EpiMono

Monomorphisms and epimorphisms in Group #

In this file, we prove monomorphisms in the category of groups are injective homomorphisms and epimorphisms are surjective homomorphisms.

theorem MonoidHom.ker_eq_bot_of_cancel {A : Type u} {B : Type v} [Group A] [Group B] {f : A →* B} (h : ∀ (u v : f.ker →* A), f.comp u = f.comp vu = v) :
f.ker =
theorem AddMonoidHom.ker_eq_bot_of_cancel {A : Type u} {B : Type v} [AddGroup A] [AddGroup B] {f : A →+ B} (h : ∀ (u v : f.ker →+ A), f.comp u = f.comp vu = v) :
f.ker =
theorem MonoidHom.range_eq_top_of_cancel {A : Type u} {B : Type v} [CommGroup A] [CommGroup B] {f : A →* B} (h : ∀ (u v : B →* B f.range), u.comp f = v.comp fu = v) :
f.range =
theorem AddMonoidHom.range_eq_top_of_cancel {A : Type u} {B : Type v} [AddCommGroup A] [AddCommGroup B] {f : A →+ B} (h : ∀ (u v : B →+ B f.range), u.comp f = v.comp fu = v) :
f.range =
instance Grp.instGroupα_1 (G : Grp) :
Group G
Equations
  • G.instGroupα_1 = G.str
instance AddGrp.instGroupα_1 (G : AddGrp) :
Equations
  • G.instGroupα_1 = G.str
inductive Grp.SurjectiveOfEpiAuxs.XWithInfinity {A B : Grp} (f : A B) :

Define X' to be the set of all left cosets with an extra point at "infinity".

Instances For
    Equations
    • One or more equations did not get rendered due to their size.
    theorem Grp.SurjectiveOfEpiAuxs.mul_smul {A B : Grp} (f : A B) (b b' : B) (x : XWithInfinity f) :
    (b * b') x = b b' x
    theorem Grp.SurjectiveOfEpiAuxs.one_smul {A B : Grp} (f : A B) (x : XWithInfinity f) :
    1 x = x
    noncomputable def Grp.SurjectiveOfEpiAuxs.tau {A B : Grp} (f : A B) :

    Let τ be the permutation on X' exchanging f.range and the point at infinity.

    Equations
    Instances For

      Let g : B ⟶ S(X') be defined as such that, for any β : B, g(β) is the function sending point at infinity to point at infinity and sending coset y to β • y.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        Define h : B ⟶ S(X') to be τ g τ⁻¹

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          The strategy is the following: assuming epi f

          theorem Grp.SurjectiveOfEpiAuxs.g_apply_fromCoset {A B : Grp} (f : A B) (x : B) (y : (Set.range fun (x : B) => x (MonoidHom.range f))) :
          ((g f) x) (XWithInfinity.fromCoset y) = XWithInfinity.fromCoset x y,
          theorem Grp.SurjectiveOfEpiAuxs.h_apply_fromCoset {A B : Grp} (f : A B) (x : B) :
          theorem Grp.SurjectiveOfEpiAuxs.h_apply_fromCoset' {A B : Grp} (f : A B) (x b : B) (hb : b MonoidHom.range f) :
          ((h f) x) (XWithInfinity.fromCoset b (MonoidHom.range f), ) = XWithInfinity.fromCoset b (MonoidHom.range f),
          theorem Grp.SurjectiveOfEpiAuxs.h_apply_fromCoset_nin_range {A B : Grp} (f : A B) (x : B) (hx : x MonoidHom.range f) (b : B) (hb : bMonoidHom.range f) :
          ((h f) x) (XWithInfinity.fromCoset b (MonoidHom.range f), ) = XWithInfinity.fromCoset (x * b) (MonoidHom.range f),
          theorem Grp.SurjectiveOfEpiAuxs.agree {A B : Grp} (f : A B) :
          (MonoidHom.range f) = {x : B | (h f) x = (g f) x}
          theorem Grp.SurjectiveOfEpiAuxs.comp_eq {A B : Grp} (f : A B) :
          CategoryTheory.CategoryStruct.comp f (let_fun this := g f; this) = CategoryTheory.CategoryStruct.comp f (let_fun this := h f; this)
          theorem Grp.SurjectiveOfEpiAuxs.g_ne_h {A B : Grp} (f : A B) (x : B) (hx : xMonoidHom.range f) :
          g f h f
          Equations
          • G.instCommGroupObjForget = G.str
          Equations
          • G.instAddCommGroupObjForget = G.str