Skip to content

Commit 925146c

Browse files
committed
chore(GroupTheory/GroupAction): split off Defs file (#18345)
The goal of this PR is to have a file with the definitions for the orbit and stabilizer of a group, and enough theory to define quotient groups.
1 parent 6c2c697 commit 925146c

File tree

16 files changed

+609
-526
lines changed

16 files changed

+609
-526
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -2951,6 +2951,7 @@ import Mathlib.GroupTheory.GroupAction.Basic
29512951
import Mathlib.GroupTheory.GroupAction.Blocks
29522952
import Mathlib.GroupTheory.GroupAction.CardCommute
29532953
import Mathlib.GroupTheory.GroupAction.ConjAct
2954+
import Mathlib.GroupTheory.GroupAction.Defs
29542955
import Mathlib.GroupTheory.GroupAction.DomAct.ActionHom
29552956
import Mathlib.GroupTheory.GroupAction.DomAct.Basic
29562957
import Mathlib.GroupTheory.GroupAction.Embedding

Mathlib/Algebra/Module/Submodule/Basic.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Nathaniel Thomas, Jeremy Avigad, Johannes Hölzl, Mario Carneiro
55
-/
66
import Mathlib.Algebra.Field.Defs
7+
import Mathlib.Algebra.Group.Subgroup.Basic
78
import Mathlib.Algebra.Group.Submonoid.Membership
9+
import Mathlib.Algebra.NoZeroSMulDivisors.Defs
810
import Mathlib.GroupTheory.GroupAction.SubMulAction
911

1012
/-!

Mathlib/CategoryTheory/Galois/GaloisObjects.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -7,6 +7,7 @@ import Mathlib.CategoryTheory.Galois.Basic
77
import Mathlib.CategoryTheory.Limits.FintypeCat
88
import Mathlib.CategoryTheory.Limits.Preserves.Limits
99
import Mathlib.CategoryTheory.Limits.Shapes.SingleObj
10+
import Mathlib.GroupTheory.GroupAction.Basic
1011
import Mathlib.Logic.Equiv.TransferInstance
1112

1213
/-!

Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,8 @@ Authors: Christian Merten
55
-/
66
import Mathlib.CategoryTheory.Limits.Types
77
import Mathlib.CategoryTheory.SingleObj
8-
import Mathlib.GroupTheory.GroupAction.Basic
8+
import Mathlib.Data.Setoid.Basic
9+
import Mathlib.GroupTheory.GroupAction.Defs
910

1011
/-!
1112
# (Co)limits of functors out of `SingleObj M`

Mathlib/Dynamics/Minimal.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,6 @@ Copyright (c) 2021 Yury Kudryashov. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yury Kudryashov
55
-/
6-
import Mathlib.GroupTheory.GroupAction.Basic
76
import Mathlib.Topology.Algebra.ConstMulAction
87

98
/-!

Mathlib/GroupTheory/Coset/Basic.lean

Lines changed: 5 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -3,9 +3,12 @@ Copyright (c) 2018 Mitchell Rowett. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Mitchell Rowett, Kim Morrison
55
-/
6-
import Mathlib.Algebra.Quotient
76
import Mathlib.Algebra.Group.Subgroup.MulOpposite
8-
import Mathlib.GroupTheory.GroupAction.Basic
7+
import Mathlib.Algebra.Quotient
8+
import Mathlib.Data.Fintype.Card
9+
import Mathlib.Data.Set.Pointwise.SMul
10+
import Mathlib.Data.Setoid.Basic
11+
import Mathlib.GroupTheory.GroupAction.Defs
912

1013
/-!
1114
# Cosets

0 commit comments

Comments
 (0)