Skip to content

Commit

Permalink
chore(Algebra/Group/Subgroup): split off Defs file (#18340)
Browse files Browse the repository at this point in the history
This PR splits off the definition of `Subgroup` and the `Group` instance into a new `Defs` file. Doing so required also moving the `Semigroup` instance on `Subsemigroup` and `Monoid` on `Submonoid` to the respective `Defs` file. So we needed to add one extra import: `Algebra.Group.InjSurj`. The imports and contents of that file are light enough in my opinion to make it worth it.




Co-authored-by: Anne Baanen <[email protected]>
  • Loading branch information
Vierkantor and Vierkantor committed Oct 28, 2024
1 parent 97a2bd1 commit 4e5fa63
Show file tree
Hide file tree
Showing 21 changed files with 932 additions and 831 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -289,6 +289,7 @@ import Mathlib.Algebra.Group.Semiconj.Defs
import Mathlib.Algebra.Group.Semiconj.Units
import Mathlib.Algebra.Group.Subgroup.Actions
import Mathlib.Algebra.Group.Subgroup.Basic
import Mathlib.Algebra.Group.Subgroup.Defs
import Mathlib.Algebra.Group.Subgroup.Finite
import Mathlib.Algebra.Group.Subgroup.MulOpposite
import Mathlib.Algebra.Group.Subgroup.Order
Expand Down
5 changes: 2 additions & 3 deletions Mathlib/Algebra/GradedMonoid.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,11 +4,10 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser
-/
import Mathlib.Algebra.BigOperators.Group.List
import Mathlib.Algebra.Group.InjSurj
import Mathlib.Algebra.Group.Action.End
import Mathlib.Algebra.Group.Submonoid.Defs
import Mathlib.Data.List.FinRange
import Mathlib.Algebra.Group.Action.Defs
import Mathlib.Data.SetLike.Basic
import Mathlib.Algebra.Group.Submonoid.Operations
import Mathlib.Data.Sigma.Basic
import Lean.Elab.Tactic

Expand Down
Loading

0 comments on commit 4e5fa63

Please sign in to comment.