Skip to content

Commit

Permalink
chore: remove some unnecessary 'open BigOperators' (#11880)
Browse files Browse the repository at this point in the history
Could we have an `open` linter, that checked for unused opened namespaces?


Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Apr 4, 2024
1 parent 6d89490 commit 16eb4bd
Show file tree
Hide file tree
Showing 13 changed files with 5 additions and 23 deletions.
2 changes: 0 additions & 2 deletions Mathlib/Algebra/Algebra/Basic.lean
Expand Up @@ -94,8 +94,6 @@ the second approach only when you need to weaken a condition on either `R` or `A

universe u v w u₁ v₁

open BigOperators

section Prio

-- We set this priority to 0 later in this file
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Algebra/Category/GroupCat/Biproducts.lean
Expand Up @@ -20,8 +20,6 @@ open CategoryTheory

open CategoryTheory.Limits

open BigOperators

universe w u

namespace AddCommGroupCat
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Algebra/CharP/Reduced.lean
Expand Up @@ -15,8 +15,6 @@ import Mathlib.RingTheory.Nilpotent

open Finset

open BigOperators

section

variable (R : Type*) [CommRing R] [IsReduced R] (p n : ℕ) [ExpChar R p]
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Lie/EngelSubalgebra.lean
Expand Up @@ -30,7 +30,7 @@ and minimal ones are nilpotent (TODO), hence Cartan subalgebras.
if it is contained in the Engel subalgebra of all its elements.
-/

open BigOperators LieAlgebra LieModule
open LieAlgebra LieModule

variable {R L M : Type*} [CommRing R] [LieRing L] [LieAlgebra R L]
[AddCommGroup M] [Module R M] [LieRingModule L M] [LieModule R L M]
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Algebra/Module/Submodule/Bilinear.lean
Expand Up @@ -29,8 +29,6 @@ universe uι u v

open Set

open BigOperators

open Pointwise

namespace Submodule
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Module/Submodule/Ker.lean
Expand Up @@ -29,7 +29,7 @@ linear algebra, vector space, module

open Function

open BigOperators Pointwise
open Pointwise

variable {R : Type*} {R₁ : Type*} {R₂ : Type*} {R₃ : Type*}
variable {K : Type*}
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Calculus/ContDiff/Defs.lean
Expand Up @@ -157,7 +157,7 @@ derivative, differentiability, higher derivative, `C^n`, multilinear, Taylor ser
noncomputable section

open scoped Classical
open BigOperators NNReal Topology Filter
open NNReal Topology Filter

local notation "∞" => (⊤ : ℕ∞)

Expand Down
3 changes: 0 additions & 3 deletions Mathlib/Analysis/Calculus/Deriv/Add.lean
Expand Up @@ -148,9 +148,6 @@ section Sum

/-! ### Derivative of a finite sum of functions -/


open BigOperators

variable {ι : Type*} {u : Finset ι} {A : ι → 𝕜 → F} {A' : ι → F}

theorem HasDerivAtFilter.sum (h : ∀ i ∈ u, HasDerivAtFilter (A i) (A' i) x L) :
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Complex/TaylorSeries.lean
Expand Up @@ -26,7 +26,7 @@ see `Complex.hasSum_taylorSeries_of_entire`, `Complex.taylorSeries_eq_of_entire`

namespace Complex

open BigOperators Nat
open Nat

variable {E : Type*} [NormedAddCommGroup E] [NormedSpace ℂ E] [CompleteSpace E] ⦃f : ℂ → E⦄

Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Analysis/Convex/Join.lean
Expand Up @@ -18,8 +18,6 @@ convex hulls of finite sets.

open Set

open BigOperators

variable {ι : Sort*} {𝕜 E : Type*}

section OrderedSemiring
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/LocallyConvex/AbsConvex.lean
Expand Up @@ -38,7 +38,7 @@ disks, convex, balanced

open NormedField Set

open BigOperators NNReal Pointwise Topology
open NNReal Pointwise Topology

variable {𝕜 E F G ι : Type*}

Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Analysis/NormedSpace/Int.lean
Expand Up @@ -19,8 +19,6 @@ The resulting nonnegative real number is denoted by `‖n‖₊`.
-/


open BigOperators

namespace Int

theorem nnnorm_coe_units (e : ℤˣ) : ‖(e : ℤ)‖₊ = 1 := by
Expand Down
3 changes: 0 additions & 3 deletions Mathlib/CategoryTheory/Linear/FunctorCategory.lean
Expand Up @@ -16,9 +16,6 @@ then `C ⥤ D` is also `R`-linear.
-/


open BigOperators

namespace CategoryTheory

open CategoryTheory.Limits Linear
Expand Down

0 comments on commit 16eb4bd

Please sign in to comment.