Documentation

Mathlib.Algebra.BigOperators.List.Lemmas

Lemmas about List.sum and List.prod requiring extra algebra imports #

theorem Commute.list_sum_right {R : Type u_8} [NonUnitalNonAssocSemiring R] (a : R) (l : List R) (h : bl, Commute a b) :
theorem Commute.list_sum_left {R : Type u_8} [NonUnitalNonAssocSemiring R] (b : R) (l : List R) (h : al, Commute a b) :
theorem List.card_nsmul_le_sum {M : Type u_3} [AddMonoid M] [Preorder M] [CovariantClass M M (Function.swap fun (x x_1 : M) => x + x_1) fun (x x_1 : M) => x x_1] [CovariantClass M M (fun (x x_1 : M) => x + x_1) fun (x x_1 : M) => x x_1] (l : List M) (n : M) (h : xl, n x) :
theorem List.pow_card_le_prod {M : Type u_3} [Monoid M] [Preorder M] [CovariantClass M M (Function.swap fun (x x_1 : M) => x * x_1) fun (x x_1 : M) => x x_1] [CovariantClass M M (fun (x x_1 : M) => x * x_1) fun (x x_1 : M) => x x_1] (l : List M) (n : M) (h : xl, n x) :
theorem List.sum_eq_zero_iff {M : Type u_3} [CanonicallyOrderedAddCommMonoid M] (l : List M) :
List.sum l = 0 xl, x = 0
theorem List.prod_eq_one_iff {M : Type u_3} [CanonicallyOrderedCommMonoid M] (l : List M) :
List.prod l = 1 xl, x = 1

If a product of integers is -1, then at least one factor must be -1.

theorem List.length_le_sum_of_one_le (L : List ) (h : iL, 1 i) :

If all elements in a list are bounded below by 1, then the length of the list is bounded by the sum of the elements.

theorem List.dvd_prod {M : Type u_3} [CommMonoid M] {a : M} {l : List M} (ha : a l) :
theorem List.dvd_sum {R : Type u_8} [NonUnitalSemiring R] {a : R} {l : List R} (h : xl, a x) :
theorem List.alternatingSum_append {α : Type u_2} [AddCommGroup α] (l₁ : List α) (l₂ : List α) :
abbrev List.alternatingSum_append.match_1 {α : Type u_1} (motive : List αList αProp) :
∀ (x x_1 : List α), (∀ (l₂ : List α), motive [] l₂)(∀ (a : α) (l₁ l₂ : List α), motive (a :: l₁) l₂)motive x x_1
Equations
  • =
Instances For
    theorem List.alternatingProd_append {α : Type u_2} [CommGroup α] (l₁ : List α) (l₂ : List α) :
    abbrev List.alternatingSum_reverse.match_1 {α : Type u_1} (motive : List αProp) :
    ∀ (x : List α), (Unitmotive [])(∀ (a : α) (l : List α), motive (a :: l))motive x
    Equations
    • =
    Instances For
      theorem List.sum_map_mul_left {ι : Type u_1} {R : Type u_8} [NonUnitalNonAssocSemiring R] (L : List ι) (f : ιR) (r : R) :
      List.sum (List.map (fun (b : ι) => r * f b) L) = r * List.sum (List.map f L)
      theorem List.sum_map_mul_right {ι : Type u_1} {R : Type u_8} [NonUnitalNonAssocSemiring R] (L : List ι) (f : ιR) (r : R) :
      List.sum (List.map (fun (b : ι) => f b * r) L) = List.sum (List.map f L) * r
      theorem MulOpposite.op_list_prod {M : Type u_3} [Monoid M] (l : List M) :
      theorem unop_map_list_prod {M : Type u_3} {N : Type u_4} [Monoid M] [Monoid N] {F : Type u_9} [FunLike F M Nᵐᵒᵖ] [MonoidHomClass F M Nᵐᵒᵖ] (f : F) (l : List M) :
      MulOpposite.unop (f (List.prod l)) = List.prod (List.reverse (List.map (MulOpposite.unop f) l))

      A morphism into the opposite monoid acts on the product by acting on the reversed elements.

      @[deprecated unop_map_list_prod]
      theorem MonoidHom.unop_map_list_prod {M : Type u_3} {N : Type u_4} [Monoid M] [Monoid N] (f : M →* Nᵐᵒᵖ) (l : List M) :
      MulOpposite.unop (f (List.prod l)) = List.prod (List.reverse (List.map (MulOpposite.unop f) l))

      A morphism into the opposite monoid acts on the product by acting on the reversed elements.