Skip to content

Commit

Permalink
chore: shake some imports (#10341)
Browse files Browse the repository at this point in the history
  • Loading branch information
sgouezel committed Feb 7, 2024
1 parent e4d4665 commit c458927
Show file tree
Hide file tree
Showing 9 changed files with 7 additions and 5 deletions.
4 changes: 1 addition & 3 deletions Mathlib/Analysis/Calculus/SmoothSeries.lean
Expand Up @@ -5,8 +5,6 @@ Authors: Sébastien Gouëzel
-/
import Mathlib.Analysis.Calculus.ContDiff.Basic
import Mathlib.Analysis.Calculus.UniformLimitsDeriv
import Mathlib.Data.Nat.Cast.WithTop
import Mathlib.RingTheory.Ideal.LocalRing
import Mathlib.Topology.Algebra.InfiniteSum.Module
import Mathlib.Analysis.NormedSpace.FunctionSeries

Expand Down Expand Up @@ -244,7 +242,7 @@ theorem contDiff_tsum (hf : ∀ i, ContDiff 𝕜 N (f i)) (hv : ∀ k : ℕ, (k
exact h'f _ _ _ hm
· intro m hm
have h'm : ((m + 1 : ℕ) : ℕ∞) ≤ N := by
simpa only [ENat.coe_add, Nat.cast_withBot, ENat.coe_one] using ENat.add_one_le_of_lt hm
simpa only [ENat.coe_add, ENat.coe_one] using ENat.add_one_le_of_lt hm
rw [iteratedFDeriv_tsum hf hv h'f hm.le]
have A :
∀ n x, HasFDerivAt (iteratedFDeriv 𝕜 m (f n)) (fderiv 𝕜 (iteratedFDeriv 𝕜 m (f n)) x) x :=
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Analysis/NormedSpace/Banach.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sébastien Gouëzel
-/
import Mathlib.Topology.MetricSpace.Baire
import Mathlib.Analysis.Normed.Group.AddTorsor
import Mathlib.Analysis.NormedSpace.OperatorNorm
import Mathlib.Analysis.NormedSpace.AffineIsometry

Expand Down
1 change: 1 addition & 0 deletions Mathlib/Analysis/NormedSpace/ContinuousAffineMap.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Oliver Nash
-/
import Mathlib.Topology.Algebra.ContinuousAffineMap
import Mathlib.Analysis.Normed.Group.AddTorsor
import Mathlib.Analysis.NormedSpace.AffineIsometry
import Mathlib.Analysis.NormedSpace.OperatorNorm

Expand Down
1 change: 1 addition & 0 deletions Mathlib/Analysis/NormedSpace/FiniteDimension.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sébastien Gouëzel
-/
import Mathlib.Analysis.Asymptotics.AsymptoticEquivalent
import Mathlib.Analysis.Normed.Group.AddTorsor
import Mathlib.Analysis.NormedSpace.AddTorsor
import Mathlib.Analysis.NormedSpace.AffineIsometry
import Mathlib.Analysis.NormedSpace.OperatorNorm
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Analysis/Seminorm.lean
Expand Up @@ -6,7 +6,6 @@ Authors: Jean Lo, Yaël Dillies, Moritz Doll
import Mathlib.Data.Real.Pointwise
import Mathlib.Analysis.Convex.Function
import Mathlib.Analysis.LocallyConvex.Basic
import Mathlib.Analysis.Normed.Group.AddTorsor
import Mathlib.Data.Real.Sqrt

#align_import analysis.seminorm from "leanprover-community/mathlib"@"09079525fd01b3dda35e96adaa08d2f943e1648c"
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Myers, Manuel Candales
-/
import Mathlib.Analysis.Convex.Between
import Mathlib.Analysis.Normed.Group.AddTorsor
import Mathlib.Geometry.Euclidean.Angle.Unoriented.Basic
import Mathlib.Analysis.NormedSpace.AffineIsometry

Expand Down
1 change: 1 addition & 0 deletions Mathlib/Geometry/Euclidean/Inversion/Basic.lean
Expand Up @@ -3,6 +3,7 @@ Copyright (c) 2022 Yury G. Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury G. Kudryashov
-/
import Mathlib.Analysis.Normed.Group.AddTorsor
import Mathlib.Analysis.InnerProductSpace.Basic

#align_import geometry.euclidean.inversion from "leanprover-community/mathlib"@"46b633fd842bef9469441c0209906f6dddd2b4f5"
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Geometry/Euclidean/PerpBisector.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov, Joseph Myers
-/
import Mathlib.Analysis.InnerProductSpace.Orthogonal
import Mathlib.Analysis.Normed.Group.AddTorsor

#align_import geometry.euclidean.basic from "leanprover-community/mathlib"@"2de9c37fa71dde2f1c6feff19876dd6a7b1519f0"

Expand Down
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2023 Kalle Kytölä. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kalle Kytölä
-/
import Mathlib.Analysis.InnerProductSpace.Basic
import Mathlib.MeasureTheory.Integral.Bochner

/-!
Expand Down

0 comments on commit c458927

Please sign in to comment.