Skip to content

Commit

Permalink
chore: remove unused variables (#18226)
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani committed Oct 25, 2024
1 parent 27e4d0a commit a4411e6
Show file tree
Hide file tree
Showing 16 changed files with 23 additions and 25 deletions.
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/Dimension/Localization.lean
Original file line number Diff line number Diff line change
Expand Up @@ -120,7 +120,7 @@ end CommRing

section Ring

variable {R} [Ring R] [IsDomain R] (S : Submonoid R)
variable {R} [Ring R] [IsDomain R]

/-- A domain that is not (left) Ore is of infinite rank.
See [cohn_1995] Proposition 1.3.6 -/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/Matrix/Circulant.lean
Original file line number Diff line number Diff line change
Expand Up @@ -32,7 +32,7 @@ circulant, matrix
-/


variable {α β m n R : Type*}
variable {α β n R : Type*}

namespace Matrix

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/RootSystem/OfBilinear.lean
Original file line number Diff line number Diff line change
Expand Up @@ -25,7 +25,7 @@ open Set Function Module

noncomputable section

variable {ι R M N : Type*} [CommRing R] [AddCommGroup M] [Module R M] [AddCommGroup N] [Module R N]
variable {R M : Type*} [CommRing R] [AddCommGroup M] [Module R M]

namespace LinearMap

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/Decomposition/RadonNikodym.lean
Original file line number Diff line number Diff line change
Expand Up @@ -88,7 +88,7 @@ lemma rnDeriv_pos' [HaveLebesgueDecomposition ν μ] [SigmaFinite μ] (hμν :

section rnDeriv_withDensity_leftRight

variable {μ ν : Measure α} {f : α → ℝ≥0∞}
variable {f : α → ℝ≥0∞}

/-- Auxiliary lemma for `rnDeriv_withDensity_left`. -/
lemma rnDeriv_withDensity_withDensity_rnDeriv_left (μ ν : Measure α) [SigmaFinite μ] [SigmaFinite ν]
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/Decomposition/SignedLebesgue.lean
Original file line number Diff line number Diff line change
Expand Up @@ -46,7 +46,7 @@ open scoped Classical MeasureTheory NNReal ENNReal

open Set

variableβ : Type*} {m : MeasurableSpace α} {μ ν : MeasureTheory.Measure α}
variable {α : Type*} {m : MeasurableSpace α} {μ : MeasureTheory.Measure α}

namespace MeasureTheory

Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -175,12 +175,10 @@ theorem AEStronglyMeasurable'.aeStronglyMeasurable'_of_measurableSpace_le_on {α
hf_ind.stronglyMeasurable_of_measurableSpace_le_on hs_m hs fun x hxs =>
Set.indicator_of_not_mem hxs _

variable {α F F' 𝕜 : Type*} {p : ℝ≥0∞} [RCLike 𝕜]
variable {α F 𝕜 : Type*} {p : ℝ≥0∞} [RCLike 𝕜]
-- 𝕜 for ℝ or ℂ
-- F for a Lp submodule
[NormedAddCommGroup F] [NormedSpace 𝕜 F]
-- F' for integrals on a Lp submodule
[NormedAddCommGroup F'] [NormedSpace 𝕜 F'] [NormedSpace ℝ F']

section LpMeas

Expand Down
4 changes: 2 additions & 2 deletions Mathlib/MeasureTheory/Measure/WithDensityVectorMeasure.lean
Original file line number Diff line number Diff line change
Expand Up @@ -26,13 +26,13 @@ noncomputable section

open scoped MeasureTheory NNReal ENNReal

variableβ : Type*} {m : MeasurableSpace α}
variable {α : Type*} {m : MeasurableSpace α}

namespace MeasureTheory

open TopologicalSpace

variableν : Measure α}
variable {μ : Measure α}
variable {E : Type*} [NormedAddCommGroup E] [NormedSpace ℝ E]

open Classical in
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/ModelTheory/Graph.lean
Original file line number Diff line number Diff line change
Expand Up @@ -21,7 +21,7 @@ This file defines first-order languages, structures, and theories in graph theor
of the theory of simple graphs.
-/

universe u v
universe u

namespace FirstOrder

Expand All @@ -31,7 +31,7 @@ open FirstOrder

open Structure

variable {α : Type u} {V : Type v} {n : ℕ}
variable {V : Type u} {n : ℕ}

/-! ### Simple Graphs -/

Expand Down
4 changes: 2 additions & 2 deletions Mathlib/ModelTheory/PartialEquiv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -40,8 +40,8 @@ namespace FirstOrder

namespace Language

variable (L : Language.{u, v}) (M : Type w) (N : Type w') {P : Type*}
variable [L.Structure M] [L.Structure N] [L.Structure P]
variable (L : Language.{u, v}) (M : Type w) (N : Type w')
variable [L.Structure M] [L.Structure N]

open FirstOrder Structure Substructure

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/NumberTheory/Cyclotomic/Gal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -152,7 +152,7 @@ end IsCyclotomicExtension

section Gal

variable [Field L] (hμ : IsPrimitiveRoot μ n) [Algebra K L] [IsCyclotomicExtension {n} K L]
variable [Field L] [Algebra K L] [IsCyclotomicExtension {n} K L]
(h : Irreducible (cyclotomic n K)) {K}

/-- `IsCyclotomicExtension.autEquivPow` repackaged in terms of `Gal`.
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/NumberTheory/Dioph.lean
Original file line number Diff line number Diff line change
Expand Up @@ -67,7 +67,7 @@ Note that this duplicates `MvPolynomial`.

section Polynomials

variable {α β γ : Type*}
variable {α β : Type*}

/-- A predicate asserting that a function is a multivariate integer polynomial.
(We are being a bit lazy here by allowing many representations for multiplication,
Expand Down Expand Up @@ -432,7 +432,7 @@ end

section

variableβ : Type} {n : ℕ}
variable {α : Type} {n : ℕ}

open Vector3

Expand Down
8 changes: 4 additions & 4 deletions Mathlib/Order/Ideal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -92,7 +92,7 @@ variable [LE P]

section

variable {I J s t : Ideal P} {x y : P}
variable {I s t : Ideal P} {x : P}

theorem toLowerSet_injective : Injective (toLowerSet : Ideal P → LowerSet P) := fun s t _ ↦ by
cases s
Expand Down Expand Up @@ -247,7 +247,7 @@ variable [Preorder P]

section

variable {I J : Ideal P} {x y : P}
variable {I : Ideal P} {x y : P}

/-- The smallest ideal containing a given element. -/
@[simps]
Expand Down Expand Up @@ -316,7 +316,7 @@ end SemilatticeSup

section SemilatticeSupDirected

variable [SemilatticeSup P] [IsDirected P (· ≥ ·)] {x : P} {I J K s t : Ideal P}
variable [SemilatticeSup P] [IsDirected P (· ≥ ·)] {x : P} {I J s t : Ideal P}

/-- The infimum of two ideals of a co-directed order is their intersection. -/
instance : Inf (Ideal P) :=
Expand Down Expand Up @@ -385,7 +385,7 @@ end SemilatticeSupDirected

section SemilatticeSupOrderBot

variable [SemilatticeSup P] [OrderBot P] {x : P} {I J K : Ideal P}
variable [SemilatticeSup P] [OrderBot P] {x : P}

instance : InfSet (Ideal P) :=
fun S ↦
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/DedekindDomain/Dvr.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,7 +43,7 @@ dedekind domain, dedekind ring
-/


variable (R A K : Type*) [CommRing R] [CommRing A] [IsDomain A] [Field K]
variable (A : Type*) [CommRing A] [IsDomain A]

open scoped nonZeroDivisors Polynomial

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/DiscreteValuationRing/TFAE.lean
Original file line number Diff line number Diff line change
Expand Up @@ -25,7 +25,7 @@ Also see `tfae_of_isNoetherianRing_of_localRing_of_isDomain` for a version witho
-/


variable (R : Type*) [CommRing R] (K : Type*) [Field K] [Algebra R K] [IsFractionRing R K]
variable (R : Type*) [CommRing R]

open scoped Multiplicative

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/PowerSeries/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -758,7 +758,7 @@ namespace Polynomial

open Finsupp Polynomial

variable {σ : Type*} {R : Type*} [CommSemiring R] (φ ψ : R[X])
variable {R : Type*} [CommSemiring R] (φ ψ : R[X])

-- Porting note: added so we can add the `@[coe]` attribute
/-- The natural inclusion from polynomials into formal power series. -/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/PowerSeries/Inverse.lean
Original file line number Diff line number Diff line change
Expand Up @@ -274,7 +274,7 @@ theorem map.isLocalHom : IsLocalHom (map f) :=
@[deprecated (since := "2024-10-10")]
alias map.isLocalRingHom := map.isLocalHom

variable [LocalRing R] [LocalRing S]
variable [LocalRing R]

instance : LocalRing R⟦X⟧ :=
{ inferInstanceAs <| LocalRing <| MvPowerSeries Unit R with }
Expand Down

0 comments on commit a4411e6

Please sign in to comment.