File tree Expand file tree Collapse file tree 1 file changed +4
-4
lines changed
Mathlib/Algebra/BigOperators/Group/List Expand file tree Collapse file tree 1 file changed +4
-4
lines changed Original file line number Diff line number Diff line change @@ -13,7 +13,7 @@ which calculate the product and sum of elements of a list
1313and `List.alternatingProd`, `List.alternatingSum`, their alternating counterparts.
1414-/
1515
16- variable {ι α β M N P G : Type *}
16+ variable {ι M N : Type *}
1717
1818namespace List
1919section Defs
@@ -42,14 +42,14 @@ end Defs
4242
4343section 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]
4848theorem 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]
5555lemma prod_induction
@@ -87,7 +87,7 @@ end MulOneClass
8787
8888section 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]
9393theorem prod_eq_foldr {l : List M} : l.prod = foldr (· * ·) 1 l := rfl
You can’t perform that action at this time.
0 commit comments