Skip to content

Commit 7e683cc

Browse files
committed
chore: remove some superfluous imports (#31616)
1 parent b0a3a60 commit 7e683cc

File tree

26 files changed

+9
-28
lines changed

26 files changed

+9
-28
lines changed

Mathlib/Algebra/Group/Basic.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,6 @@ import Mathlib.Algebra.Group.Defs
88
import Mathlib.Data.Int.Init
99
import Mathlib.Logic.Function.Iterate
1010
import Mathlib.Tactic.SimpRw
11-
import Mathlib.Tactic.SplitIfs
1211

1312
/-!
1413
# Basic lemmas about semigroups, monoids, and groups

Mathlib/Algebra/Group/Center.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -3,11 +3,9 @@ Copyright (c) 2021 Eric Wieser. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Eric Wieser, Jireh Loreaux
55
-/
6-
import Mathlib.Algebra.Group.Commute.Units
76
import Mathlib.Algebra.Group.Invertible.Basic
8-
import Mathlib.Logic.Basic
9-
import Mathlib.Data.Set.Basic
107
import Mathlib.Algebra.Notation.Prod
8+
import Mathlib.Data.Set.Basic
119

1210
/-!
1311
# Centers of magmas and semigroups

Mathlib/Algebra/Group/Defs.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,6 @@ import Mathlib.Algebra.Notation.Defs
88
import Mathlib.Algebra.Regular.Defs
99
import Mathlib.Data.Int.Notation
1010
import Mathlib.Data.Nat.BinaryRec
11-
import Mathlib.Logic.Function.Defs
1211
import Mathlib.Tactic.MkIffOfInductiveProp
1312
import Mathlib.Tactic.OfNat
1413
import Mathlib.Tactic.Basic

Mathlib/Algebra/Group/Finsupp.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,6 @@ import Mathlib.Algebra.Group.Equiv.Defs
77
import Mathlib.Algebra.Group.Pi.Lemmas
88
import Mathlib.Data.Finset.Max
99
import Mathlib.Data.Finsupp.Single
10-
import Mathlib.Tactic.FastInstance
1110

1211
/-!
1312
# Additive monoid structure on `ι →₀ M`

Mathlib/Algebra/Group/Nat/Hom.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -3,8 +3,6 @@ Copyright (c) 2020 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.Algebra.Group.Equiv.Defs
7-
import Mathlib.Algebra.Group.Hom.Basic
86
import Mathlib.Algebra.Group.Nat.Defs
97
import Mathlib.Algebra.Group.TypeTags.Hom
108
import Mathlib.Tactic.Spread

Mathlib/Algebra/GroupWithZero/Defs.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,6 @@ Authors: Johan Commelin
55
-/
66
import Mathlib.Algebra.Group.Defs
77
import Mathlib.Logic.Nontrivial.Defs
8-
import Mathlib.Tactic.SplitIfs
98
import Mathlib.Logic.Basic
109

1110
/-!

Mathlib/Algebra/Opposites.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,6 @@ Authors: Kenny Lau
66
import Mathlib.Algebra.Group.Defs
77
import Mathlib.Logic.Equiv.Defs
88
import Mathlib.Logic.Nontrivial.Basic
9-
import Mathlib.Logic.IsEmpty
109

1110
/-!
1211
# Multiplicative opposite and algebraic operations on it

Mathlib/Algebra/Order/GroupWithZero/Canonical.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -14,6 +14,7 @@ import Mathlib.Algebra.Order.Monoid.Basic
1414
import Mathlib.Algebra.Order.Monoid.OrderDual
1515
import Mathlib.Algebra.Order.Monoid.TypeTags
1616
import Mathlib.Algebra.Group.WithOne.Map
17+
import Mathlib.Tactic.Tauto
1718

1819
/-!
1920
# Linearly ordered commutative groups and monoids with a zero element adjoined

Mathlib/Algebra/Order/Quantale.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,6 @@ Copyright (c) 2024 Pieter Cuijpers. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Pieter Cuijpers
55
-/
6-
import Mathlib.Algebra.Group.Defs
76
import Mathlib.Algebra.Order.Monoid.Unbundled.Basic
87
import Mathlib.Order.CompleteLattice.Basic
98
import Mathlib.Tactic.Variable

Mathlib/Algebra/PEmptyInstances.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: Julian Kuelshammer
55
-/
66
import Mathlib.Algebra.Group.Defs
7-
import Mathlib.Tactic.ToAdditive
87

98
/-!
109
# Instances on pempty

0 commit comments

Comments
 (0)