Skip to content
Closed
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
2 changes: 0 additions & 2 deletions Mathlib/Algebra/Category/AlgCat/Monoidal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,8 +43,6 @@ noncomputable abbrev tensorHom {W X Y Z : AlgCat.{u} R} (f : W ⟶ X) (g : Y ⟶
tensorObj W Y ⟶ tensorObj X Z :=
ofHom <| Algebra.TensorProduct.map f.hom g.hom

open MonoidalCategory

end instMonoidalCategory

open instMonoidalCategory
Expand Down
5 changes: 0 additions & 5 deletions Mathlib/Algebra/Group/Equiv/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -28,11 +28,6 @@ open Function

variable {F α β M M₁ M₂ M₃ N N₁ N₂ N₃ P Q G H : Type*}

namespace EmbeddingLike
variable [One M] [One N] [FunLike F M N] [EmbeddingLike F M N] [OneHomClass F M N]

end EmbeddingLike

variable [EquivLike F α β]

@[to_additive]
Expand Down
26 changes: 0 additions & 26 deletions Mathlib/Algebra/Group/Pointwise/Finset/Scalar.lean
Original file line number Diff line number Diff line change
Expand Up @@ -340,39 +340,13 @@ theorem op_smul_finset_smul_eq_smul_smul_finset (a : α) (s : Finset β) (t : Fi

end SMul


section IsRightCancelMul

variable [Mul α] [IsRightCancelMul α] [DecidableEq α] {s t : Finset α} {a : α}


end IsRightCancelMul

section CancelMonoid
variable [DecidableEq α] [CancelMonoid α] {s : Finset α} {m n : ℕ}


end CancelMonoid

section Group
variable [Group α] [DecidableEq α] {s t : Finset α}


end Group

@[to_additive]
theorem image_smul_comm [DecidableEq β] [DecidableEq γ] [SMul α β] [SMul α γ] (f : β → γ) (a : α)
(s : Finset β) : (∀ b, f (a • b) = a • f b) → (a • s).image f = a • s.image f :=
image_comm

end Finset

namespace Fintype
variable {ι : Type*} {α β : ι → Type*} [Fintype ι] [DecidableEq ι] [∀ i, DecidableEq (β i)]
[∀ i, DecidableEq (α i)]

end Fintype

open Pointwise

namespace Set
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Algebra/Group/Subgroup/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -403,8 +403,6 @@ theorem _root_.normalizerCondition_iff_only_full_group_self_normalizing :
simp only [lt_iff_le_and_ne, le_normalizer, le_top, Ne]
tauto

variable (H)

end Normalizer

end Subgroup
Expand Down
6 changes: 0 additions & 6 deletions Mathlib/Algebra/Group/Submonoid/Membership.lean
Original file line number Diff line number Diff line change
Expand Up @@ -42,12 +42,6 @@ assert_not_exists MonoidWithZero

variable {M A B : Type*}

section Assoc

variable [Monoid M] [SetLike B M] [SubmonoidClass B M] {S : B}

end Assoc

section NonAssoc

variable [MulOneClass M]
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Algebra/GroupWithZero/Units/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -133,8 +133,6 @@ theorem inverse_zero : inverse (0 : M₀) = 0 := by
nontriviality
exact inverse_non_unit _ not_isUnit_zero

variable {M₀}

end Ring

theorem IsUnit.ringInverse {a : M₀} : IsUnit a → IsUnit (Ring.inverse a)
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Algebra/Module/RingHom.lean
Original file line number Diff line number Diff line change
Expand Up @@ -63,8 +63,6 @@ abbrev Module.compHom [Semiring S] (f : S →+* R) : Module S M :=
-- TODO(jmc): there should be a rw-lemma `smul_comp` close to `SMulZeroClass.compFun`
add_smul := fun r s x => show f (r + s) • x = f r • x + f s • x by simp [add_smul] }

variable {M}

end AddCommMonoid

/-- A ring homomorphism `f : R →+* M` defines a module structure by `r • x = f r * x`.
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1344,8 +1344,6 @@ lemma zpow_lt_zpow_iff_left₀ (ha : 0 ≤ a) (hb : 0 ≤ b) (hn : 0 < n) : a ^

end MulPosMono

variable [MulPosStrictMono G₀]

end GroupWithZero.LinearOrder

section CommGroupWithZero
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/AlgebraicGeometry/AffineScheme.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1216,8 +1216,6 @@ lemma specTargetImageFactorization_comp :
specTargetImageFactorization f ≫ Spec.map (specTargetImageRingHom f) = f :=
f.liftQuotient_comp _ _

open RingHom

end Factorization

section Stalks
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -399,8 +399,6 @@ instance : hoFunctor₂.{u}.Monoidal :=
instance hoFunctor.monoidal : hoFunctor.{u}.Monoidal :=
inferInstanceAs (truncation 2 ⋙ hoFunctor₂).Monoidal

open MonoidalCategory

end Truncated

/-- An equivalence between the vertices of a simplicial set `X` and the
Expand Down
4 changes: 0 additions & 4 deletions Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean
Original file line number Diff line number Diff line change
Expand Up @@ -187,8 +187,6 @@ theorem superpolynomialDecay_const_mul_iff [ContinuousMul β] {c : β} (hc0 : c
fun h => (h.const_mul c⁻¹).congr fun x => by simp [← mul_assoc, inv_mul_cancel₀ hc0], fun h =>
h.const_mul c⟩

variable {l k f}

end Field

section LinearOrderedField
Expand Down Expand Up @@ -272,8 +270,6 @@ theorem superpolynomialDecay_mul_param_pow_iff (hk : Tendsto k l atTop) (n : ℕ
SuperpolynomialDecay l k (f * k ^ n) ↔ SuperpolynomialDecay l k f := by
simpa [mul_comm f] using superpolynomialDecay_param_pow_mul_iff f hk n

variable {f}

end LinearOrderedField

section NormedLinearOrderedField
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean
Original file line number Diff line number Diff line change
Expand Up @@ -459,8 +459,6 @@ theorem y_support {D : ℝ} (Dpos : 0 < D) (D_lt_one : D < 1) :
⟨fun _ hx => (y_pos_of_mem_ball Dpos D_lt_one hx).ne', fun _ hx =>
y_eq_zero_of_notMem_ball Dpos hx⟩

variable {E}

end HelperDefinitions

instance (priority := 100) {E : Type*} [NormedAddCommGroup E] [NormedSpace ℝ E]
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Analysis/Calculus/LineDeriv/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -451,8 +451,6 @@ theorem norm_lineDeriv_le_of_lipschitz {f : E → F} {x₀ : E}
{C : ℝ≥0} (hlip : LipschitzWith C f) : ‖lineDeriv 𝕜 f x₀ v‖ ≤ C * ‖v‖ :=
norm_lineDeriv_le_of_lipschitzOn 𝕜 univ_mem (lipschitzOnWith_univ.2 hlip)

variable {𝕜}

end NormedSpace

section Zero
Expand Down
5 changes: 0 additions & 5 deletions Mathlib/Analysis/Convex/Cone/InnerDual.lean
Original file line number Diff line number Diff line change
Expand Up @@ -186,11 +186,6 @@ theorem ConvexCone.hyperplane_separation_of_nonempty_of_isClosed_of_notMem (K :
_ = ⟪b - z, b - z + z⟫_ℝ := (inner_add_right _ _ _).symm
_ = ⟪b - z, b⟫_ℝ := by rw [sub_add_cancel]

namespace ProperCone
variable {F : Type*} [NormedAddCommGroup F] [InnerProductSpace ℝ F]

end ProperCone

end CompleteSpace

end Dual
2 changes: 0 additions & 2 deletions Mathlib/Analysis/Distribution/SchwartzSpace.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1227,8 +1227,6 @@ theorem toBoundedContinuousFunctionCLM_apply (f : 𝓢(E, F)) (x : E) :
toBoundedContinuousFunctionCLM 𝕜 E F f x = f x :=
rfl

variable {E}

end BoundedContinuousFunction

section ZeroAtInfty
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Analysis/Normed/Module/Alternating/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -365,8 +365,6 @@ def restrictScalarsLI : E [⋀^ι]→L[𝕜] F →ₗᵢ[𝕜'] E [⋀^ι]→L[
map_smul' _ _ := rfl
norm_map' _ := rfl

variable {𝕜'}

end restrictScalars

/-- The difference `f m₁ - f m₂` is controlled in terms of `‖f‖` and `‖m₁ - m₂‖`, precise version.
Expand Down
6 changes: 0 additions & 6 deletions Mathlib/CategoryTheory/Limits/Shapes/IsTerminal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -334,12 +334,6 @@ theorem InitialMonoClass.of_isTerminal {I T : C} (hI : IsInitial I) (hT : IsTerm
(_ : Mono (hI.to T)) : InitialMonoClass C :=
InitialMonoClass.of_isInitial hI fun X => mono_of_mono_fac (hI.hom_ext (_ ≫ hT.from X) (hI.to T))

section Comparison

variable {D : Type u₂} [Category.{v₂} D] (G : C ⥤ D)

end Comparison

variable {J : Type u} [Category.{v} J]

/-- From a functor `F : J ⥤ C`, given an initial object of `J`, construct a cone for `J`.
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/CategoryTheory/Noetherian.lean
Original file line number Diff line number Diff line change
Expand Up @@ -45,6 +45,4 @@ class Artinian : Prop extends EssentiallySmall C where

attribute [instance] Artinian.isArtinianObject

open Subobject

end CategoryTheory
2 changes: 0 additions & 2 deletions Mathlib/CategoryTheory/Sites/Canonical.lean
Original file line number Diff line number Diff line change
Expand Up @@ -229,8 +229,6 @@ theorem isSheaf_of_isRepresentable {J : GrothendieckTopology C} [Subcanonical J]
(P : Cᵒᵖ ⥤ Type v) [P.IsRepresentable] : Presieve.IsSheaf J P :=
Presieve.isSheaf_of_le _ J.le_canonical (Sheaf.isSheaf_of_isRepresentable P)

variable {J : GrothendieckTopology C}

end Subcanonical

variable (J : GrothendieckTopology C)
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Control/LawfulFix.lean
Original file line number Diff line number Diff line change
Expand Up @@ -165,8 +165,6 @@ theorem fix_eq_of_ωScottContinuous (hc : ωScottContinuous g) :
intro i
exists i.succ

variable {f}

end Part

namespace Part
Expand Down
6 changes: 0 additions & 6 deletions Mathlib/Data/Matrix/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -157,12 +157,6 @@ end Diag

open Matrix

section AddCommMonoid

variable [AddCommMonoid α] [Mul α]

end AddCommMonoid

section NonAssocSemiring

variable [NonAssocSemiring α]
Expand Down
4 changes: 0 additions & 4 deletions Mathlib/Data/Matrix/Mul.lean
Original file line number Diff line number Diff line change
Expand Up @@ -472,8 +472,6 @@ theorem op_smul_one_eq_diagonal [DecidableEq m] (a : α) :
MulOpposite.op a • (1 : Matrix m m α) = diagonal fun _ => a := by
simp_rw [← diagonal_one, ← diagonal_smul, Pi.smul_def, op_smul_eq_mul, one_mul]

variable (α n)

end NonAssocSemiring

section NonUnitalSemiring
Expand Down Expand Up @@ -1152,8 +1150,6 @@ theorem transpose_mul [AddCommMonoid α] [CommMagma α] [Fintype n] (M : Matrix
ext
apply dotProduct_comm

variable (m n α)

end Transpose

theorem submatrix_mul [Fintype n] [Fintype o] [Mul α] [AddCommMonoid α] {p q : Type*}
Expand Down
10 changes: 0 additions & 10 deletions Mathlib/Data/Tree/RBMap.lean
Original file line number Diff line number Diff line change
Expand Up @@ -21,13 +21,3 @@ Implement a `Traversable` instance for `Tree`.
<https://leanprover-community.github.io/archive/stream/113488-general/topic/tactic.20question.html>
-/
Copy link
Collaborator

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I'm guessing this file should be deprecated, but not here

Copy link
Collaborator Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Yes, I wanted to fix enough to make the linter compliant and leave everything else for later PRs.

Copy link
Collaborator

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

#34043 deprecates the module


public section

namespace Tree

universe u

variable {α : Type u}

end Tree
6 changes: 0 additions & 6 deletions Mathlib/GroupTheory/Congruence/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -505,12 +505,6 @@ theorem comap_rel {f : M → N} (H : ∀ x y, f (x * y) = f x * f y) {c : Con N}
comap f H c x y ↔ c (f x) (f y) :=
Iff.rfl

section

open Quotient

end

end

section MulOneClass
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -155,8 +155,6 @@ variable (K V)
instance finiteDimensional_bot : FiniteDimensional K (⊥ : Submodule K V) :=
.of_rank_eq_zero <| by simp

variable {K V}

end ZeroRank

namespace Submodule
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -53,8 +53,6 @@ abbrev tensorHom {W X Y Z : QuadraticModuleCat.{u} R} (f : W ⟶ X) (g : Y ⟶ Z
tensorObj W Y ⟶ tensorObj X Z :=
⟨f.toIsometry.tmul g.toIsometry⟩

open MonoidalCategory

end instMonoidalCategory

open instMonoidalCategory
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/LinearAlgebra/TensorAlgebra/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -316,8 +316,6 @@ def tprod (n : ℕ) : MultilinearMap R (fun _ : Fin n => M) (TensorAlgebra R M)
theorem tprod_apply {n : ℕ} (x : Fin n → M) : tprod R M n x = (List.ofFn fun i => ι R (x i)).prod :=
rfl

variable {R M}

end TensorAlgebra

namespace FreeAlgebra
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean
Original file line number Diff line number Diff line change
Expand Up @@ -115,8 +115,6 @@ theorem ae_eq_zero_of_forall_dual [NormedAddCommGroup E] [NormedSpace 𝕜 E]
ae_eq_zero_of_forall_dual_of_isSeparable 𝕜 (.of_separableSpace Set.univ) hf
(Eventually.of_forall fun _ => Set.mem_univ _)

variable {𝕜}

end AeEqOfForall

variable {α E : Type*} {m m0 : MeasurableSpace α} {μ : Measure α}
Expand Down
4 changes: 0 additions & 4 deletions Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -695,8 +695,6 @@ def coeToLp : Lp.simpleFunc E p μ →L[𝕜] Lp E p μ :=
map_smul' := fun _ _ => rfl
cont := Lp.simpleFunc.uniformContinuous.continuous }

variable {α E 𝕜}

end CoeToLp

section Order
Expand Down Expand Up @@ -789,8 +787,6 @@ theorem denseRange_coeSimpleFuncNonnegToLpNonneg [hp : Fact (1 ≤ p)] (hp_ne_to
exact h_toLp n
· rfl

variable {p μ G}

end Order

end simpleFunc
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/MeasureTheory/Integral/Prod.lean
Original file line number Diff line number Diff line change
Expand Up @@ -162,8 +162,6 @@ theorem integrable_measure_prodMk_left {s : Set (α × β)} (hs : MeasurableSet

end Measure

open Measure

end MeasureTheory

open MeasureTheory.Measure
Expand Down
7 changes: 4 additions & 3 deletions Mathlib/NumberTheory/Padics/PadicNumbers.lean
Original file line number Diff line number Diff line change
Expand Up @@ -321,12 +321,13 @@ end Valuation

end PadicSeq

-- Porting note: Commented out `padic_index_simp` tactic

/-
section

open PadicSeq

-- Porting note: Commented out `padic_index_simp` tactic
/-
private unsafe def index_simp_core (hh hf hg : expr)
(at_ : Interactive.Loc := Interactive.Loc.ns [none]) : tactic Unit := do
let [v1, v2, v3] ← [hh, hf, hg].mapM fun n => tactic.mk_app `` stationary_point [n] <|> return n
Expand All @@ -344,9 +345,9 @@ unsafe def tactic.interactive.padic_index_simp (l : interactive.parse interactiv
(at_ : interactive.parse interactive.types.location) : tactic Unit := do
let [h, f, g] ← l.mapM tactic.i_to_expr
index_simp_core h f g at_
-/

end
-/

namespace PadicSeq

Expand Down
7 changes: 0 additions & 7 deletions Mathlib/Order/Filter/AtTopBot/Monoid.lean
Original file line number Diff line number Diff line change
Expand Up @@ -171,11 +171,4 @@ theorem Tendsto.atBot_of_mul_const_le (hg : ∃ C, ∀ x, C ≤ g x)

end OrderedCancelCommMonoid

section OrderedCancelAddCommMonoid

variable [AddCommMonoid M] [PartialOrder M] [IsOrderedCancelAddMonoid M]
{l : Filter α} {f g : α → M}

end OrderedCancelAddCommMonoid

end Filter
Loading
Loading