Skip to content

Commit 9e5cdbf

Browse files
committed
chore(CategoryTheory/Limits/Types): split Shapes.lean (#31258)
The file `CategoryTheory.Limits.Types.Shapes` is split in several files corresponding to different kinds of shapes of limits/colimits. (As that constructions are not self-dual, dual shapes appear in separate files, e.g. `Pushouts` and `Pullbacks`.)
1 parent e6df210 commit 9e5cdbf

File tree

29 files changed

+1147
-1025
lines changed

29 files changed

+1147
-1025
lines changed

Mathlib.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -2597,14 +2597,20 @@ import Mathlib.CategoryTheory.Limits.Shapes.ZeroObjects
25972597
import Mathlib.CategoryTheory.Limits.Sifted
25982598
import Mathlib.CategoryTheory.Limits.Skeleton
25992599
import Mathlib.CategoryTheory.Limits.SmallComplete
2600+
import Mathlib.CategoryTheory.Limits.Types.Coequalizers
26002601
import Mathlib.CategoryTheory.Limits.Types.ColimitType
26012602
import Mathlib.CategoryTheory.Limits.Types.ColimitTypeFiltered
26022603
import Mathlib.CategoryTheory.Limits.Types.Colimits
2604+
import Mathlib.CategoryTheory.Limits.Types.Coproducts
2605+
import Mathlib.CategoryTheory.Limits.Types.Equalizers
26032606
import Mathlib.CategoryTheory.Limits.Types.Filtered
26042607
import Mathlib.CategoryTheory.Limits.Types.Images
26052608
import Mathlib.CategoryTheory.Limits.Types.Limits
26062609
import Mathlib.CategoryTheory.Limits.Types.Multicoequalizer
2610+
import Mathlib.CategoryTheory.Limits.Types.Multiequalizer
2611+
import Mathlib.CategoryTheory.Limits.Types.Products
26072612
import Mathlib.CategoryTheory.Limits.Types.Pullbacks
2613+
import Mathlib.CategoryTheory.Limits.Types.Pushouts
26082614
import Mathlib.CategoryTheory.Limits.Types.Shapes
26092615
import Mathlib.CategoryTheory.Limits.Types.Yoneda
26102616
import Mathlib.CategoryTheory.Limits.Unit

Mathlib/Algebra/Category/Grp/Adjunctions.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,8 @@ Authors: Kim Morrison, Johannes Hölzl
55
-/
66
import Mathlib.Algebra.Category.Grp.Preadditive
77
import Mathlib.GroupTheory.FreeAbelianGroup
8-
import Mathlib.CategoryTheory.Limits.Types.Shapes
8+
import Mathlib.CategoryTheory.Adjunction.Limits
9+
import Mathlib.CategoryTheory.Limits.Types.Coproducts
910

1011
/-!
1112
# Adjunctions regarding the category of (abelian) groups

Mathlib/AlgebraicGeometry/GluingOneHypercover.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -5,6 +5,7 @@ Authors: Calle Sönne, Joël Riou, Ravi Vakil
55
-/
66
import Mathlib.AlgebraicGeometry.Gluing
77
import Mathlib.AlgebraicGeometry.Sites.BigZariski
8+
import Mathlib.CategoryTheory.Limits.Types.Multiequalizer
89
import Mathlib.CategoryTheory.Sites.Hypercover.One
910

1011
/-!

Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johan Commelin, Kim Morrison, Adam Topaz, Joël Riou
55
-/
66
import Mathlib.AlgebraicTopology.SimplicialSet.NerveNondegenerate
7-
import Mathlib.CategoryTheory.Limits.Types.Shapes
87
import Mathlib.Data.Fin.VecNotation
98
import Mathlib.Order.Fin.SuccAboveOrderIso
109

Mathlib/CategoryTheory/Extensive.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,9 @@ Authors: Andrew Yang
55
-/
66
import Mathlib.CategoryTheory.Limits.Shapes.Pullback.CommSq
77
import Mathlib.CategoryTheory.Limits.Shapes.StrictInitial
8-
import Mathlib.CategoryTheory.Limits.Types.Shapes
8+
import Mathlib.CategoryTheory.Limits.Types.Coproducts
9+
import Mathlib.CategoryTheory.Limits.Types.Products
10+
import Mathlib.CategoryTheory.Limits.Types.Pullbacks
911
import Mathlib.Topology.Category.TopCat.Limits.Pullbacks
1012
import Mathlib.CategoryTheory.Limits.FunctorCategory.Basic
1113
import Mathlib.CategoryTheory.Limits.Constructions.FiniteProductsOfBinaryProducts

Mathlib/CategoryTheory/Galois/Basic.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -9,6 +9,7 @@ import Mathlib.CategoryTheory.Limits.FintypeCat
99
import Mathlib.CategoryTheory.Limits.MonoCoprod
1010
import Mathlib.CategoryTheory.Limits.Shapes.ConcreteCategory
1111
import Mathlib.CategoryTheory.Limits.Shapes.Diagonal
12+
import Mathlib.CategoryTheory.Limits.Types.Equalizers
1213
import Mathlib.CategoryTheory.SingleObj
1314
import Mathlib.Data.Finite.Card
1415

Mathlib/CategoryTheory/GlueData.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,7 @@ import Mathlib.Tactic.CategoryTheory.Elementwise
77
import Mathlib.CategoryTheory.Limits.Shapes.Multiequalizer
88
import Mathlib.CategoryTheory.Limits.Constructions.EpiMono
99
import Mathlib.CategoryTheory.Limits.Preserves.Limits
10-
import Mathlib.CategoryTheory.Limits.Types.Shapes
10+
import Mathlib.CategoryTheory.Limits.Types.Coproducts
1111

1212
/-!
1313
# Gluing data

Mathlib/CategoryTheory/Limits/FilteredColimitCommutesProduct.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -4,9 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Markus Himmel
55
-/
66
import Mathlib.CategoryTheory.Limits.FunctorCategory.Filtered
7-
import Mathlib.CategoryTheory.Limits.Types.Filtered
8-
import Mathlib.CategoryTheory.Limits.Types.Shapes
97
import Mathlib.CategoryTheory.Limits.FunctorCategory.Shapes.Products
8+
import Mathlib.CategoryTheory.Limits.Types.Filtered
9+
import Mathlib.CategoryTheory.Limits.Types.Products
1010

1111
/-!
1212
# The IPC property

Mathlib/CategoryTheory/Limits/Final.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,7 @@ import Mathlib.CategoryTheory.Category.Cat.AsSmall
77
import Mathlib.CategoryTheory.Comma.StructuredArrow.Basic
88
import Mathlib.CategoryTheory.IsConnected
99
import Mathlib.CategoryTheory.Limits.Preserves.Shapes.Terminal
10-
import Mathlib.CategoryTheory.Limits.Types.Shapes
10+
import Mathlib.CategoryTheory.Limits.Types.Products
1111
import Mathlib.CategoryTheory.Limits.Shapes.Grothendieck
1212
import Mathlib.CategoryTheory.Filtered.Basic
1313
import Mathlib.CategoryTheory.Limits.Yoneda

Mathlib/CategoryTheory/Limits/FintypeCat.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,9 +4,12 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Christian Merten
55
-/
66
import Mathlib.CategoryTheory.FintypeCat
7+
import Mathlib.CategoryTheory.Limits.Creates
78
import Mathlib.CategoryTheory.Limits.Preserves.Finite
89
import Mathlib.CategoryTheory.Limits.Preserves.Shapes.Products
9-
import Mathlib.CategoryTheory.Limits.Types.Shapes
10+
import Mathlib.CategoryTheory.Limits.Types.Colimits
11+
import Mathlib.CategoryTheory.Limits.Types.Limits
12+
import Mathlib.CategoryTheory.Limits.Types.Products
1013
import Mathlib.Data.Finite.Prod
1114
import Mathlib.Data.Finite.Sigma
1215

0 commit comments

Comments
 (0)