Skip to content

Commit 38e09f6

Browse files
committed
chore (BigOperators.Finsupp): avoid importing Order.BigOperators.Ring.Finset (#14336)
This is one part of the import path from `Algebra.Order.Group.Defs` here and clearly unnecessary.
1 parent 1462590 commit 38e09f6

File tree

10 files changed

+12
-7
lines changed

10 files changed

+12
-7
lines changed

Mathlib/Algebra/BigOperators/Finsupp.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,6 @@ Authors: Kenny Lau
55
-/
66
import Mathlib.Algebra.BigOperators.Pi
77
import Mathlib.Algebra.BigOperators.Ring
8-
import Mathlib.Algebra.Order.BigOperators.Ring.Finset
98
import Mathlib.Algebra.BigOperators.Fin
109
import Mathlib.Algebra.Group.Submonoid.Membership
1110
import Mathlib.Data.Finsupp.Fin
@@ -691,9 +690,10 @@ namespace Nat
691690

692691
-- Porting note: Needed to replace pow with (· ^ ·)
693692
/-- If `0 : ℕ` is not in the support of `f : ℕ →₀ ℕ` then `0 < ∏ x ∈ f.support, x ^ (f x)`. -/
694-
theorem prod_pow_pos_of_zero_not_mem_support {f : ℕ →₀ ℕ} (hf : 0 ∉ f.support) :
693+
theorem prod_pow_pos_of_zero_not_mem_support {f : ℕ →₀ ℕ} (nhf : 0 ∉ f.support) :
695694
0 < f.prod (· ^ ·) :=
696-
Finset.prod_pos fun a ha => pos_iff_ne_zero.mpr (pow_ne_zero _ fun H => by subst H; exact hf ha)
695+
Nat.pos_iff_ne_zero.mpr <| Finset.prod_ne_zero_iff.mpr fun _ hf =>
696+
pow_ne_zero _ fun H => by subst H; exact nhf hf
697697
#align nat.prod_pow_pos_of_zero_not_mem_support Nat.prod_pow_pos_of_zero_not_mem_support
698698

699699
end Nat

Mathlib/Algebra/MvPolynomial/Degrees.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,6 @@ Authors: Johannes Hölzl, Johan Commelin, Mario Carneiro
55
-/
66
import Mathlib.Algebra.MonoidAlgebra.Degree
77
import Mathlib.Algebra.MvPolynomial.Rename
8-
import Mathlib.Algebra.Order.BigOperators.Ring.Finset
98

109
#align_import data.mv_polynomial.variables from "leanprover-community/mathlib"@"2f5b500a507264de86d666a5f87ddb976e2d8de4"
1110

Mathlib/Algebra/Order/Antidiag/Finsupp.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -5,6 +5,7 @@ Authors: Antoine Chambert-Loir, María Inés de Frutos-Fernández, Eric Wieser,
55
Yaël Dillies
66
-/
77
import Mathlib.Algebra.Order.Antidiag.Pi
8+
import Mathlib.Algebra.Order.BigOperators.Group.Finset
89
import Mathlib.Data.Finsupp.Basic
910

1011
/-!

Mathlib/Analysis/Convex/Basic.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ Copyright (c) 2019 Alexander Bentkamp. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Alexander Bentkamp, Yury Kudriashov, Yaël Dillies
55
-/
6+
import Mathlib.Algebra.Order.BigOperators.Ring.Finset
67
import Mathlib.Algebra.Order.Module.OrderedSMul
78
import Mathlib.Analysis.Convex.Star
89
import Mathlib.LinearAlgebra.AffineSpace.AffineSubspace

Mathlib/Analysis/Convex/Segment.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -388,7 +388,7 @@ theorem mem_openSegment_iff_div : x ∈ openSegment 𝕜 y z ↔
388388
use a, b, ha, hb
389389
rw [hab, div_one, div_one]
390390
· rintro ⟨a, b, ha, hb, rfl⟩
391-
have hab : 0 < a + b := by positivity
391+
have hab : 0 < a + b := add_pos' ha hb
392392
refine ⟨a / (a + b), b / (a + b), by positivity, by positivity, ?_, rfl⟩
393393
rw [← add_div, div_self hab.ne']
394394
#align mem_open_segment_iff_div mem_openSegment_iff_div

Mathlib/Combinatorics/Optimization/ValuedCSP.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: Martin Dvorak
55
-/
66
import Mathlib.Algebra.BigOperators.Fin
7+
import Mathlib.Algebra.Order.BigOperators.Group.Multiset
78
import Mathlib.Data.Fin.VecNotation
89
import Mathlib.Data.Matrix.Notation
910

Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean

Lines changed: 1 addition & 2 deletions
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: Adrian Wüthrich
55
-/
66
import Mathlib.Combinatorics.SimpleGraph.AdjMatrix
7-
import Mathlib.Data.Real.StarOrdered
87
import Mathlib.LinearAlgebra.Matrix.PosDef
98

109
/-!
@@ -88,7 +87,7 @@ theorem lapMatrix_toLinearMap₂' [Field R] [CharZero R] (x : V → R) :
8887
ring_nf
8988

9089
/-- The Laplacian matrix is positive semidefinite -/
91-
theorem posSemidef_lapMatrix [LinearOrderedField R] [StarRing R] [StarOrderedRing R]
90+
theorem posSemidef_lapMatrix [LinearOrderedField R] [StarRing R]
9291
[TrivialStar R] : PosSemidef (G.lapMatrix R) := by
9392
constructor
9493
· rw [IsHermitian, conjTranspose_eq_transpose_of_trivial, isSymm_lapMatrix]

Mathlib/LinearAlgebra/Matrix/AbsoluteValue.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ Copyright (c) 2021 Anne Baanen. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Anne Baanen
55
-/
6+
import Mathlib.Algebra.Order.BigOperators.Ring.Finset
67
import Mathlib.Data.Int.AbsoluteValue
78
import Mathlib.LinearAlgebra.Matrix.Determinant.Basic
89

Mathlib/NumberTheory/Primorial.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: Patrick Stevens, Yury Kudryashov
55
-/
66
import Mathlib.Algebra.BigOperators.Associated
7+
import Mathlib.Algebra.Order.BigOperators.Ring.Finset
78
import Mathlib.Algebra.Order.Ring.Abs
89
import Mathlib.Data.Nat.Choose.Sum
910
import Mathlib.Data.Nat.Choose.Dvd

scripts/noshake.json

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -333,6 +333,8 @@
333333
"Mathlib.Analysis.InnerProductSpace.Basic":
334334
["Mathlib.Algebra.Module.LinearMap.Basic"],
335335
"Mathlib.Analysis.Distribution.SchwartzSpace": ["Mathlib.Tactic.MoveAdd"],
336+
"Mathlib.Analysis.Convex.Basic":
337+
["Mathlib.Algebra.Order.BigOperators.Ring.Finset"],
336338
"Mathlib.AlgebraicTopology.DoldKan.Notations":
337339
["Mathlib.AlgebraicTopology.AlternatingFaceMapComplex"],
338340
"Mathlib.Algebra.Star.Module": ["Mathlib.Algebra.Module.LinearMap.Star"],

0 commit comments

Comments
 (0)