Skip to content

Commit

Permalink
chore(GroupTheory/QuotientGroup): split off Defs file (#18348)
Browse files Browse the repository at this point in the history
The goal of this PR is to have a file with the definitions for the quotient of a group by a normal subgroup.
  • Loading branch information
Vierkantor committed Oct 29, 2024
1 parent 43e571a commit 8a2a571
Show file tree
Hide file tree
Showing 16 changed files with 317 additions and 271 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3007,6 +3007,7 @@ import Mathlib.GroupTheory.Perm.ViaEmbedding
import Mathlib.GroupTheory.PresentedGroup
import Mathlib.GroupTheory.PushoutI
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.GroupTheory.QuotientGroup.Defs
import Mathlib.GroupTheory.QuotientGroup.Finite
import Mathlib.GroupTheory.Schreier
import Mathlib.GroupTheory.SchurZassenhaus
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/Grp/Colimits.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@ import Mathlib.Algebra.Category.Grp.Preadditive
import Mathlib.CategoryTheory.Limits.Shapes.Kernels
import Mathlib.CategoryTheory.Limits.Shapes.FiniteLimits
import Mathlib.CategoryTheory.ConcreteCategory.Elementwise
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.GroupTheory.QuotientGroup.Defs

/-!
# The category of additive commutative groups has all colimits.
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Algebra/Category/Grp/EpiMono.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,8 @@ Authors: Jujian Zhang
import Mathlib.Algebra.Category.Grp.EquivalenceGroupAddGroup
import Mathlib.CategoryTheory.ConcreteCategory.EpiMono
import Mathlib.CategoryTheory.Limits.Constructions.EpiMono
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.GroupTheory.Coset.Basic
import Mathlib.GroupTheory.QuotientGroup.Defs

/-!
# Monomorphisms and epimorphisms in `Group`
Expand Down
4 changes: 3 additions & 1 deletion Mathlib/Algebra/CharZero/Quotient.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,8 +4,10 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser
-/
import Mathlib.Algebra.Field.Basic
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.Algebra.Group.Subgroup.ZPowers
import Mathlib.Algebra.Order.Group.Unbundled.Int
import Mathlib.Algebra.Module.Defs
import Mathlib.GroupTheory.QuotientGroup.Defs

/-!
# Lemmas about quotients in characteristic zero
Expand Down
5 changes: 3 additions & 2 deletions Mathlib/Algebra/ModEq.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,11 +3,12 @@ Copyright (c) 2023 Yaël Dillies. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import Mathlib.Data.Int.ModEq
import Mathlib.Algebra.Field.Basic
import Mathlib.Algebra.Group.Subgroup.ZPowers
import Mathlib.Algebra.NoZeroSMulDivisors.Basic
import Mathlib.Algebra.Order.Ring.Int
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.Data.Int.ModEq
import Mathlib.GroupTheory.QuotientGroup.Defs

/-!
# Equality modulo an element
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Pointwise/Stabilizer.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import Mathlib.Algebra.Group.Pointwise.Finset.Basic
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.GroupTheory.QuotientGroup.Defs

/-!
# Stabilizer of a set under a pointwise action
Expand Down
5 changes: 3 additions & 2 deletions Mathlib/GroupTheory/Abelianization.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,9 +4,10 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kenny Lau, Michael Howes
-/
import Mathlib.Data.Finite.Card
import Mathlib.GroupTheory.Finiteness
import Mathlib.GroupTheory.Commutator.Basic
import Mathlib.Data.Finite.Prod
import Mathlib.GroupTheory.Commutator.Basic
import Mathlib.GroupTheory.Coset.Basic
import Mathlib.GroupTheory.Finiteness

/-!
# The abelianization of a group
Expand Down
5 changes: 3 additions & 2 deletions Mathlib/GroupTheory/Coxeter/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,12 +3,13 @@ Copyright (c) 2024 Newell Jensen. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Newell Jensen, Mitchell Lee
-/
import Mathlib.Algebra.Group.Subgroup.Pointwise
import Mathlib.Algebra.Ring.Int
import Mathlib.GroupTheory.PresentedGroup
import Mathlib.GroupTheory.Coxeter.Matrix
import Mathlib.GroupTheory.PresentedGroup
import Mathlib.Tactic.NormNum.DivMod
import Mathlib.Tactic.Ring
import Mathlib.Tactic.Use
import Mathlib.Tactic.NormNum.DivMod

/-!
# Coxeter groups and Coxeter systems
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/GroupTheory/Divisible.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jujian Zhang
-/
import Mathlib.Algebra.Group.ULift
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.Algebra.Group.Subgroup.Pointwise
import Mathlib.GroupTheory.QuotientGroup.Defs
import Mathlib.Tactic.NormNum.Eq

/-!
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/GroupTheory/Finiteness.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,9 @@ Copyright (c) 2021 Riccardo Brasca. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Riccardo Brasca
-/
import Mathlib.Algebra.Group.Subgroup.Pointwise
import Mathlib.Data.Set.Pointwise.Finite
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.GroupTheory.QuotientGroup.Defs
import Mathlib.SetTheory.Cardinal.Finite

/-!
Expand Down
1 change: 1 addition & 0 deletions Mathlib/GroupTheory/Index.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,7 @@ import Mathlib.Data.Set.Card
import Mathlib.GroupTheory.Coset.Card
import Mathlib.GroupTheory.Finiteness
import Mathlib.GroupTheory.GroupAction.Quotient
import Mathlib.GroupTheory.QuotientGroup.Basic

/-!
# Index of a Subgroup
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/PresentedGroup.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Michael Howes, Newell Jensen
-/
import Mathlib.GroupTheory.FreeGroup.Basic
import Mathlib.GroupTheory.QuotientGroup.Basic
import Mathlib.GroupTheory.QuotientGroup.Defs

/-!
# Defining a group given by generators and relations
Expand Down
Loading

0 comments on commit 8a2a571

Please sign in to comment.