Skip to content

Commit c0ae1f3

Browse files
chore: remove some unused variables (#31017)
1 parent aa78411 commit c0ae1f3

File tree

1 file changed

+4
-4
lines changed
  • Mathlib/Algebra/BigOperators/Group/List

1 file changed

+4
-4
lines changed

Mathlib/Algebra/BigOperators/Group/List/Defs.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ which calculate the product and sum of elements of a list
1313
and `List.alternatingProd`, `List.alternatingSum`, their alternating counterparts.
1414
-/
1515

16-
variableα β M N P G : Type*}
16+
variable {ι M N : Type*}
1717

1818
namespace List
1919
section Defs
@@ -42,14 +42,14 @@ end Defs
4242

4343
section Mul
4444

45-
variable [Mul M] [One M] {l : List M} {a : M}
45+
variable [Mul M] [One M] {a : M} {l : List M}
4646

4747
@[to_additive existing, simp]
4848
theorem prod_nil : ([] : List M).prod = 1 :=
4949
rfl
5050

5151
@[to_additive existing, simp]
52-
theorem prod_cons {a} {l : List M} : (a :: l).prod = a * l.prod := rfl
52+
theorem prod_cons : (a :: l).prod = a * l.prod := rfl
5353

5454
@[to_additive]
5555
lemma prod_induction
@@ -87,7 +87,7 @@ end MulOneClass
8787

8888
section Monoid
8989

90-
variable [Monoid M] [Monoid N] [Monoid P] {l l₁ l₂ : List M} {a : M}
90+
variable [Monoid M] [Monoid N]
9191

9292
@[to_additive]
9393
theorem prod_eq_foldr {l : List M} : l.prod = foldr (· * ·) 1 l := rfl

0 commit comments

Comments
 (0)