Skip to content

Commit 2ed7908

Browse files
committed
chore: unused arguments (#17348)
1 parent c8c6a5f commit 2ed7908

File tree

953 files changed

+2726
-2472
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

953 files changed

+2726
-2472
lines changed

Mathlib/Algebra/Algebra/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -479,8 +479,8 @@ def LinearMap.extendScalarsOfSurjectiveEquiv (h : Function.Surjective (algebraMa
479479
map_add' _ _ := rfl
480480
map_smul' _ _ := rfl
481481
invFun f := f.restrictScalars S
482-
left_inv f := rfl
483-
right_inv f := rfl
482+
left_inv _ := rfl
483+
right_inv _ := rfl
484484

485485
/-- If `R →+* S` is surjective, then `R`-linear maps are also `S`-linear. -/
486486
abbrev LinearMap.extendScalarsOfSurjective (h : Function.Surjective (algebraMap R S))

Mathlib/Algebra/Algebra/Equiv.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -625,10 +625,10 @@ end OfRingEquiv
625625
-- @[simps (config := .lemmasOnly) one]
626626
instance aut : Group (A₁ ≃ₐ[R] A₁) where
627627
mul ϕ ψ := ψ.trans ϕ
628-
mul_assoc ϕ ψ χ := rfl
628+
mul_assoc _ _ _ := rfl
629629
one := refl
630-
one_mul ϕ := ext fun x => rfl
631-
mul_one ϕ := ext fun x => rfl
630+
one_mul _ := ext fun _ => rfl
631+
mul_one _ := ext fun _ => rfl
632632
inv := symm
633633
inv_mul_cancel ϕ := ext <| symm_apply_apply ϕ
634634

Mathlib/Algebra/Algebra/Hom.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -354,10 +354,10 @@ protected theorem map_list_prod (s : List A) : φ s.prod = (s.map φ).prod :=
354354
@[simps (config := .lemmasOnly) toSemigroup_toMul_mul toOne_one]
355355
instance End : Monoid (A →ₐ[R] A) where
356356
mul := comp
357-
mul_assoc ϕ ψ χ := rfl
357+
mul_assoc _ _ _ := rfl
358358
one := AlgHom.id R A
359-
one_mul ϕ := rfl
360-
mul_one ϕ := rfl
359+
one_mul _ := rfl
360+
mul_one _ := rfl
361361

362362
@[simp]
363363
theorem one_apply (x : A) : (1 : A →ₐ[R] A) x = x :=

Mathlib/Algebra/Algebra/Operations.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -490,10 +490,10 @@ submodules. -/
490490
def equivOpposite : Submodule R Aᵐᵒᵖ ≃+* (Submodule R A)ᵐᵒᵖ where
491491
toFun p := op <| p.comap (↑(opLinearEquiv R : A ≃ₗ[R] Aᵐᵒᵖ) : A →ₗ[R] Aᵐᵒᵖ)
492492
invFun p := p.unop.comap (↑(opLinearEquiv R : A ≃ₗ[R] Aᵐᵒᵖ).symm : Aᵐᵒᵖ →ₗ[R] A)
493-
left_inv p := SetLike.coe_injective <| rfl
494-
right_inv p := unop_injective <| SetLike.coe_injective rfl
493+
left_inv _ := SetLike.coe_injective <| rfl
494+
right_inv _ := unop_injective <| SetLike.coe_injective rfl
495495
map_add' p q := by simp [comap_equiv_eq_map_symm, ← op_add]
496-
map_mul' p q := congr_arg op <| comap_op_mul _ _
496+
map_mul' _ _ := congr_arg op <| comap_op_mul _ _
497497

498498
protected theorem map_pow {A'} [Semiring A'] [Algebra R A'] (f : A →ₐ[R] A') (n : ℕ) :
499499
map f.toLinearMap (M ^ n) = map f.toLinearMap M ^ n :=
@@ -647,7 +647,7 @@ theorem mem_div_iff_smul_subset {x : A} {I J : Submodule R A} : x ∈ I / J ↔
647647
fun h y ⟨y', hy', xy'_eq_y⟩ => by
648648
rw [← xy'_eq_y]
649649
apply h
650-
assumption, fun h y hy => h (Set.smul_mem_smul_set hy)⟩
650+
assumption, fun h _ hy => h (Set.smul_mem_smul_set hy)⟩
651651

652652
theorem le_div_iff {I J K : Submodule R A} : I ≤ J / K ↔ ∀ x ∈ I, ∀ z ∈ K, x * z ∈ J :=
653653
Iff.refl _

Mathlib/Algebra/Algebra/Opposite.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -38,7 +38,7 @@ variable [IsScalarTower R S A]
3838
namespace MulOpposite
3939

4040
instance instAlgebra : Algebra R Aᵐᵒᵖ where
41-
toRingHom := (algebraMap R A).toOpposite fun x y => Algebra.commutes _ _
41+
toRingHom := (algebraMap R A).toOpposite fun _ _ => Algebra.commutes _ _
4242
smul_def' c x := unop_injective <| by
4343
simp only [unop_smul, RingHom.toOpposite_apply, Function.comp_apply, unop_mul, op_mul,
4444
Algebra.smul_def, Algebra.commutes, op_unop, unop_op]

Mathlib/Algebra/Algebra/Subalgebra/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -280,8 +280,8 @@ instance (priority := 500) algebra' [CommSemiring R'] [SMul R' R] [Algebra R' A]
280280
Algebra.algebraMap_eq_smul_one]
281281
exact algebraMap_mem S
282282
_ with
283-
commutes' := fun c x => Subtype.eq <| Algebra.commutes _ _
284-
smul_def' := fun c x => Subtype.eq <| Algebra.smul_def _ _ }
283+
commutes' := fun _ _ => Subtype.eq <| Algebra.commutes _ _
284+
smul_def' := fun _ _ => Subtype.eq <| Algebra.smul_def _ _ }
285285

286286
instance algebra : Algebra R S := S.algebra'
287287

Mathlib/Algebra/Algebra/Tower.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -265,7 +265,7 @@ open IsScalarTower
265265

266266
theorem smul_mem_span_smul_of_mem {s : Set S} {t : Set A} {k : S} (hks : k ∈ span R s) {x : A}
267267
(hx : x ∈ t) : k • x ∈ span R (s • t) :=
268-
span_induction hks (fun c hc => subset_span <| Set.smul_mem_smul hc hx)
268+
span_induction hks (fun _ hc => subset_span <| Set.smul_mem_smul hc hx)
269269
(by rw [zero_smul]; exact zero_mem _)
270270
(fun c₁ c₂ ih₁ ih₂ => by rw [add_smul]; exact add_mem ih₁ ih₂)
271271
fun b c hc => by rw [IsScalarTower.smul_assoc]; exact smul_mem _ _ hc
@@ -274,7 +274,7 @@ theorem span_smul_of_span_eq_top {s : Set S} (hs : span R s = ⊤) (t : Set A) :
274274
span R (s • t) = (span S t).restrictScalars R :=
275275
le_antisymm
276276
(span_le.2 fun _x ⟨p, _hps, _q, hqt, hpqx⟩ ↦ hpqx ▸ (span S t).smul_mem p (subset_span hqt))
277-
fun p hp ↦ closure_induction hp (zero_mem _) (fun _ _ ↦ add_mem) fun s0 y hy ↦ by
277+
fun _ hp ↦ closure_induction hp (zero_mem _) (fun _ _ ↦ add_mem) fun s0 y hy ↦ by
278278
refine span_induction (hs ▸ mem_top : s0 ∈ span R s)
279279
(fun x hx ↦ subset_span ⟨x, hx, y, hy, rfl⟩) ?_ ?_ ?_
280280
· rw [zero_smul]; apply zero_mem

Mathlib/Algebra/Algebra/ZMod.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -32,7 +32,7 @@ abbrev algebra' (h : m ∣ n) : Algebra (ZMod n) R :=
3232
rcases ZMod.intCast_surjective a with ⟨k, rfl⟩
3333
show ZMod.castHom h R k * r = r * ZMod.castHom h R k
3434
rw [map_intCast, Int.cast_comm]
35-
smul_def' := fun a r => rfl }
35+
smul_def' := fun _ _ => rfl }
3636

3737
end
3838

Mathlib/Algebra/Associated/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -831,7 +831,7 @@ instance instCommMonoid : CommMonoid (Associates M) where
831831
instance instPreorder : Preorder (Associates M) where
832832
le := Dvd.dvd
833833
le_refl := dvd_refl
834-
le_trans a b c := dvd_trans
834+
le_trans _ _ _ := dvd_trans
835835

836836
/-- `Associates.mk` as a `MonoidHom`. -/
837837
protected def mkMonoidHom : M →* Associates M where

Mathlib/Algebra/BigOperators/Associated.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -187,7 +187,7 @@ variable [CancelCommMonoidWithZero α]
187187

188188
theorem exists_mem_multiset_le_of_prime {s : Multiset (Associates α)} {p : Associates α}
189189
(hp : Prime p) : p ≤ s.prod → ∃ a ∈ s, p ≤ a :=
190-
Multiset.induction_on s (fund, Eq⟩ => (hp.ne_one (mul_eq_one.1 Eq.symm).1).elim)
190+
Multiset.induction_on s (fun_, Eq⟩ => (hp.ne_one (mul_eq_one.1 Eq.symm).1).elim)
191191
fun a s ih h =>
192192
have : p ≤ a * s.prod := by simpa using h
193193
match Prime.le_or_le hp this with

0 commit comments

Comments
 (0)