Skip to content

Commit

Permalink
chore(Algebra/Group/Subgroup): split Lattice, Map, Ker from `Ba…
Browse files Browse the repository at this point in the history
…sic.lean` (#19295)

The file `Algebra/Group/Subgroup/Basic.lean` is very long. Following the design of the `Submodule` folder, split it into:
* `Lattice.lean`: `CompleteLattice` instance, `Subgroup.closure`
* `Map.lean`: `Subgroup.map`, `Subgroup.comap`
* `Ker.lean`: `MonoidHom.ker`, `MonoidHom.range` and `MonoidHom.eqLocus`
  • Loading branch information
Vierkantor committed Nov 21, 2024
1 parent 1d199de commit e4a142c
Show file tree
Hide file tree
Showing 23 changed files with 1,623 additions and 1,421 deletions.
3 changes: 3 additions & 0 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -298,6 +298,9 @@ 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.Ker
import Mathlib.Algebra.Group.Subgroup.Lattice
import Mathlib.Algebra.Group.Subgroup.Map
import Mathlib.Algebra.Group.Subgroup.MulOpposite
import Mathlib.Algebra.Group.Subgroup.MulOppositeLemmas
import Mathlib.Algebra.Group.Subgroup.Order
Expand Down
Loading

0 comments on commit e4a142c

Please sign in to comment.