Skip to content

Commit f4c4ca6

Browse files
committed
chore: reduce imports (leanprover-community#9830)
This uses the improved `shake` script from leanprover-community#9772 to reduce imports across mathlib. The corresponding `noshake.json` file has been added to leanprover-community#9772. Co-authored-by: Mario Carneiro <[email protected]>
1 parent e29e9b5 commit f4c4ca6

File tree

583 files changed

+573
-512
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

583 files changed

+573
-512
lines changed

Archive/Wiedijk100Theorems/PerfectNumbers.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -7,6 +7,7 @@ import Mathlib.NumberTheory.ArithmeticFunction
77
import Mathlib.NumberTheory.LucasLehmer
88
import Mathlib.Algebra.GeomSum
99
import Mathlib.RingTheory.Multiplicity
10+
import Mathlib.Tactic.NormNum.Prime
1011

1112
#align_import wiedijk_100_theorems.perfect_numbers from "leanprover-community/mathlib"@"5563b1b49e86e135e8c7b556da5ad2f5ff881cad"
1213

Counterexamples/Cyclotomic105.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Riccardo Brasca
55
-/
66
import Mathlib.RingTheory.Polynomial.Cyclotomic.Basic
7+
import Mathlib.Tactic.NormNum.Prime
78

89
#align_import cyclotomic_105 from "leanprover-community/mathlib"@"328375597f2c0dd00522d9c2e5a33b6a6128feeb"
910

Counterexamples/DirectSumIsInternal.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -5,6 +5,7 @@ Authors: Eric Wieser, Kevin Buzzard
55
-/
66
import Mathlib.Algebra.DirectSum.Module
77
import Mathlib.Algebra.Group.ConjFinite
8+
import Mathlib.Data.Fintype.Lattice
89
import Mathlib.Tactic.FinCases
910

1011
#align_import direct_sum_is_internal from "leanprover-community/mathlib"@"328375597f2c0dd00522d9c2e5a33b6a6128feeb"

Mathlib/Algebra/Algebra/Bilinear.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: Kenny Lau, Yury Kudryashov
55
-/
66
import Mathlib.Algebra.Algebra.Basic
7-
import Mathlib.Algebra.Algebra.Equiv
87
import Mathlib.Algebra.Algebra.NonUnitalHom
98
import Mathlib.Algebra.GroupPower.IterateHom
109
import Mathlib.LinearAlgebra.TensorProduct

Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Jireh Loreaux
55
-/
66
import Mathlib.Algebra.Algebra.NonUnitalHom
77
import Mathlib.Data.Set.UnionLift
8-
import Mathlib.LinearAlgebra.Finsupp
8+
import Mathlib.LinearAlgebra.Span
99
import Mathlib.RingTheory.NonUnitalSubring.Basic
1010

1111
/-!

Mathlib/Algebra/BigOperators/Basic.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -11,6 +11,7 @@ import Mathlib.Data.Finset.Sigma
1111
import Mathlib.Data.Finset.Sum
1212
import Mathlib.Data.Fintype.Pi
1313
import Mathlib.Data.Int.Cast.Lemmas
14+
import Mathlib.Data.Set.Image
1415

1516
#align_import algebra.big_operators.basic from "leanprover-community/mathlib"@"65a1391a0106c9204fe45bc73a039f056558cb83"
1617

Mathlib/Algebra/BigOperators/Fin.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -7,6 +7,7 @@ import Mathlib.Data.Fintype.BigOperators
77
import Mathlib.Data.Fintype.Fin
88
import Mathlib.Data.List.FinRange
99
import Mathlib.Logic.Equiv.Fin
10+
import Mathlib.Algebra.BigOperators.Ring
1011

1112
#align_import algebra.big_operators.fin from "leanprover-community/mathlib"@"cc5dd6244981976cc9da7afc4eee5682b037a013"
1213

Mathlib/Algebra/BigOperators/Multiset/Basic.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ Copyright (c) 2015 Microsoft Corporation. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Mario Carneiro
55
-/
6+
import Mathlib.Algebra.Order.Group.Abs
67
import Mathlib.Data.List.BigOperators.Basic
78
import Mathlib.Data.Multiset.Basic
89

Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,6 @@ Copyright (c) 2023 Eric Wieser. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Eric Wieser
55
-/
6-
import Mathlib.CategoryTheory.Monoidal.Braided
76
import Mathlib.CategoryTheory.Monoidal.Transport
87
import Mathlib.Algebra.Category.AlgebraCat.Basic
98
import Mathlib.Algebra.Category.ModuleCat.Monoidal.Basic

Mathlib/Algebra/Category/GroupCat/Biproducts.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -7,6 +7,7 @@ import Mathlib.Algebra.Group.Pi
77
import Mathlib.Algebra.Category.GroupCat.Preadditive
88
import Mathlib.CategoryTheory.Preadditive.Biproducts
99
import Mathlib.Algebra.Category.GroupCat.Limits
10+
import Mathlib.Tactic.CategoryTheory.Elementwise
1011

1112
#align_import algebra.category.Group.biproducts from "leanprover-community/mathlib"@"234ddfeaa5572bc13716dd215c6444410a679a8e"
1213

0 commit comments

Comments
 (0)