Skip to content

Commit

Permalink
precise docstrings
Browse files Browse the repository at this point in the history
  • Loading branch information
YaelDillies committed Nov 27, 2024
1 parent 8ea6f6e commit cde1831
Showing 1 changed file with 11 additions and 13 deletions.
24 changes: 11 additions & 13 deletions Mathlib/GroupTheory/Goursat.lean
Original file line number Diff line number Diff line change
Expand Up @@ -13,8 +13,8 @@ import Mathlib.GroupTheory.QuotientGroup.Defs
This file proves Goursat's lemma for subgroups.
If `I` is a subgroup of `G × H` which projects fully on both factors, then there exist normal
subgroups `G' ≤ G` and `H' ≤ H` such that the image of `I` in `G ⧸ G' × H ⧸ H'` is the graph of an
isomorphism `G ⧸ G' ≃ H ⧸ H'`.
subgroups `G' ≤ G` and `H' ≤ H` such that `G' × H' ≤ I` and the image of `I` in `G ⧸ G' × H ⧸ H'` is
the graph of an isomorphism `G ⧸ G' ≃ H ⧸ H'`.
`G'` and `H'` can be explicitly constructed as `Subgroup.goursatFst I` and `Subgroup.goursatSnd I`
respectively.
Expand Down Expand Up @@ -83,16 +83,16 @@ lemma goursatFst_prod_goursatSnd_le : I.goursatFst.prod I.goursatSnd ≤ I := by
/-- **Goursat's lemma** for a subgroup of with surjective projections.
If `I` is a subgroup of `G × H` which projects fully on both factors, then there exist normal
subgroups `M ≤ G` and `N ≤ H` such that the image of `I` in `G ⧸ M × H ⧸ N` is the graph of an
isomorphism `G ⧸ M ≃ H ⧸ N'`.
subgroups `M ≤ G` and `N ≤ H` such that `G' × H' ≤ I` and the image of `I` in `G ⧸ M × H ⧸ N` is the
graph of an isomorphism `G ⧸ M ≃ H ⧸ N'`.
`G'` and `H'` can be explicitly constructed as `I.goursatFst` and `I.goursatSnd` respectively. -/
@[to_additive
"**Goursat's lemma** for a subgroup of with surjective projections.
If `I` is a subgroup of `G × H` which projects fully on both factors, then there exist normal
subgroups `M ≤ G` and `N ≤ H` such that the image of `I` in `G ⧸ M × H ⧸ N` is the graph of an
isomorphism `G ⧸ M ≃ H ⧸ N'`.
subgroups `M ≤ G` and `N ≤ H` such that `G' × H' ≤ I` and the image of `I` in `G ⧸ M × H ⧸ N` is the
graph of an isomorphism `G ⧸ M ≃ H ⧸ N'`.
`G'` and `H'` can be explicitly constructed as `I.goursatFst` and `I.goursatSnd` respectively."]
lemma goursat_surjective :
Expand All @@ -111,16 +111,14 @@ lemma goursat_surjective :
/-- **Goursat's lemma** for an arbitrary subgroup.
If `I` is a subgroup of `G × H`, then there exist subgroups `G' ≤ G`, `H' ≤ H` and normal subgroups
`M ≤ G'` and `N ≤ H'` such that the image of `I` in `G' ⧸ M × H' ⧸ N` is the graph of an
isomorphism `G ⧸ G' ≃ H ⧸ H'`. -/
`M ≤ G'` and `N ≤ H'` such that `M × N ≤ I` and the image of `I` in `G' ⧸ M × H' ⧸ N` is the graph
of an isomorphism `G ⧸ G' ≃ H ⧸ H'`. -/
@[to_additive
"**Goursat's lemma** for an arbitrary subgroup.
If `I` is a subgroup of `G × H` which projects fully on both factors, then there exist normal
subgroups `G' ≤ G` and `H' ≤ H` such that the image of `I` in `G ⧸ G' × H ⧸ H'` is the graph of an
isomorphism `G ⧸ G' ≃ H ⧸ H'`.
`G'` and `H'` can be explicitly constructed as `I.goursatFst` and `I.goursatSnd` respectively."]
If `I` is a subgroup of `G × H`, then there exist subgroups `G' ≤ G`, `H' ≤ H` and normal subgroups
`M ≤ G'` and `N ≤ H'` such that `M × N ≤ I` and the image of `I` in `G' ⧸ M × H' ⧸ N` is the graph
of an isomorphism `G ⧸ G' ≃ H ⧸ H'`."]
lemma goursat :
∃ (G' : Subgroup G) (H' : Subgroup H) (M : Subgroup G') (N : Subgroup H') (_ : M.Normal)
(_ : N.Normal) (e : G' ⧸ M ≃* H' ⧸ N),
Expand Down

0 comments on commit cde1831

Please sign in to comment.