Loogle!
Result
Found 3287 declarations mentioning Finset.sum. Of these, only the first 200 are shown.
- Finset.sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : M - Finset.sum_val ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{M : Type u_3} [AddCommMonoid M] (s : Finset M) : s.val.sum = s.sum id - Finset.sum.eq_1 ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : s.sum f = (Multiset.map f s.val).sum - Finset.sum_multiset_singleton ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} (s : Finset ฮน) : โ a โ s, {a} = s.val - Finset.sum_eq_multiset_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : โ x โ s, f x = (Multiset.map f s.val).sum - Finset.sum_map_val ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : (Multiset.map f s.val).sum = โ a โ s, f a - Finset.sum_mk ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Multiset ฮน) (hs : s.Nodup) (f : ฮน โ M) : { val := s, nodup := hs }.sum f = (Multiset.map f s).sum - Finset.sum_empty' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] : โ .sum = fun x => 0 - Finset.op_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : MulOpposite.op (โ x โ s, f x) = โ x โ s, MulOpposite.op (f x) - Finset.sum_empty ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} {f : ฮน โ M} [AddCommMonoid M] : โ x โ โ , f x = 0 - Finset.sum_of_isEmpty ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} {f : ฮน โ M} [AddCommMonoid M] [IsEmpty ฮน] (s : Finset ฮน) : โ i โ s, f i = 0 - Finset.sum_range_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{M : Type u_3} [AddCommMonoid M] (f : โ โ M) : โ k โ Finset.range 0, f k = 0 - Finset.unop_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ Mแตแตแต) : MulOpposite.unop (โ x โ s, f x) = โ x โ s, MulOpposite.unop (f x) - Multiset.card_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮฑ : Type u_6} (s : Finset ฮน) (f : ฮน โ Multiset ฮฑ) : (โ i โ s, f i).card = โ i โ s, (f i).card - Finset.nonempty_of_sum_ne_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} {s : Finset ฮน} {f : ฮน โ M} [AddCommMonoid M] (h : โ x โ s, f x โ 0) : s.Nonempty - Fintype.sum_empty ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [Fintype ฮน] [AddCommMonoid M] [IsEmpty ฮน] (f : ฮน โ M) : โ x, f x = 0 - Finset.sum_toList ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{M : Type u_7} [AddCommMonoid M] (s : Finset M) : s.toList.sum = โ x โ s, x - Function.Bijective.sum_comp ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [Fintype ฮน] [Fintype ฮบ] [AddCommMonoid M] {e : ฮน โ ฮบ} (he : Function.Bijective e) (g : ฮบ โ M) : โ i, g (e i) = โ i, g i - Multiset.count_sum' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮฑ : Type u_6} [DecidableEq ฮฑ] {s : Finset ฮน} {a : ฮฑ} {f : ฮน โ Multiset ฮฑ} : Multiset.count a (โ x โ s, f x) = โ x โ s, Multiset.count a (f x) - Finset.sum_const_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} {s : Finset ฮน} [AddCommMonoid M] : โ _x โ s, 0 = 0 - Finset.sum_filter_count_eq_countP ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} [DecidableEq ฮน] (p : ฮน โ Prop) [DecidablePred p] (l : List ฮน) : โ x โ l.toFinset with p x, List.count x l = List.countP (fun b => decide (p b)) l - Finset.sum_map_toList ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : (List.map f s.toList).sum = s.sum f - Finset.sum_map' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (e : ฮน โช ฮบ) : (Finset.map e s).sum = fun f => โ x โ s, f (e x) - Finset.sum_map ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (e : ฮน โช ฮบ) (f : ฮบ โ M) : โ x โ Finset.map e s, f x = โ x โ s, f (e x) - Finset.sum_int_mod ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} (s : Finset ฮน) (n : โค) (f : ฮน โ โค) : (โ i โ s, f i) % n = (โ i โ s, f i % n) % n - Finset.sum_nat_mod ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} (s : Finset ฮน) (n : โ) (f : ฮน โ โ) : (โ i โ s, f i) % n = (โ i โ s, f i % n) % n - Multiset.disjoint_finset_sum_left ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮฑ : Type u_6} {i : Finset ฮน} {f : ฮน โ Multiset ฮฑ} {a : Multiset ฮฑ} : Disjoint (i.sum f) a โ โ b โ i, Disjoint (f b) a - Multiset.disjoint_finset_sum_right ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮฑ : Type u_6} {i : Finset ฮน} {f : ฮน โ Multiset ฮฑ} {a : Multiset ฮฑ} : Disjoint a (i.sum f) โ โ b โ i, Disjoint a (f b) - Finset.sum_ite_index ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (p : Prop) [Decidable p] (s t : Finset ฮน) (f : ฮน โ M) : โ x โ if p then s else t, f x = if p then โ x โ s, f x else โ x โ t, f x - Finset.sum_ite_irrel ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (p : Prop) [Decidable p] (s : Finset ฮน) (f g : ฮน โ M) : (โ x โ s, if p then f x else g x) = if p then โ x โ s, f x else โ x โ s, g x - Fintype.sum_bijective ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [Fintype ฮน] [Fintype ฮบ] [AddCommMonoid M] (e : ฮน โ ฮบ) (he : Function.Bijective e) (f : ฮน โ M) (g : ฮบ โ M) (h : โ (x : ฮน), f x = g (e x)) : โ x, f x = โ x, g x - Function.Bijective.finset_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [Fintype ฮน] [Fintype ฮบ] [AddCommMonoid M] (e : ฮน โ ฮบ) (he : Function.Bijective e) (f : ฮน โ M) (g : ฮบ โ M) (h : โ (x : ฮน), f x = g (e x)) : โ x, f x = โ x, g x - Finset.sum_neg_distrib ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {G : Type u_5} {s : Finset ฮน} [SubtractionCommMonoid G] (f : ฮน โ G) : โ x โ s, -f x = -โ x โ s, f x - Equiv.sum_comp ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [Fintype ฮน] [Fintype ฮบ] [AddCommMonoid M] (e : ฮน โ ฮบ) (g : ฮบ โ M) : โ i, g (e i) = โ i, g i - Finset.sum_nsmul ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (n : โ) (f : ฮน โ M) : โ x โ s, n โข f x = n โข โ x โ s, f x - Finset.sum_induction_nonempty ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {s : Finset ฮน} {M : Type u_7} [AddCommMonoid M] (f : ฮน โ M) (p : M โ Prop) (hom : โ (a b : M), p a โ p b โ p (a + b)) (nonempty : s.Nonempty) (base : โ x โ s, p (f x)) : p (โ x โ s, f x) - Finset.sum_zsmul ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {G : Type u_5} [SubtractionCommMonoid G] (f : ฮน โ G) (s : Finset ฮน) (n : โค) : โ a โ s, n โข f a = n โข โ a โ s, f a - Finset.sum_dite_irrel ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (p : Prop) [Decidable p] (s : Finset ฮน) (f : p โ ฮน โ M) (g : ยฌp โ ฮน โ M) : (โ x โ s, if h : p then f h x else g h x) = if h : p then โ x โ s, f h x else โ x โ s, g h x - Fintype.sum_equiv ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [Fintype ฮน] [Fintype ฮบ] [AddCommMonoid M] (e : ฮน โ ฮบ) (f : ฮน โ M) (g : ฮบ โ M) (h : โ (x : ฮน), f x = g (e x)) : โ x, f x = โ x, g x - Finset.ite_sum_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (p : Prop) [Decidable p] (s : Finset ฮน) (f : ฮน โ M) : (if p then โ x โ s, f x else 0) = โ x โ s, if p then f x else 0 - Finset.ite_zero_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (p : Prop) [Decidable p] (s : Finset ฮน) (f : ฮน โ M) : (if p then 0 else โ x โ s, f x) = โ x โ s, if p then 0 else f x - map_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} {N : Type u_4} [AddCommMonoid M] [AddCommMonoid N] {G : Type u_7} [FunLike G M N] [AddMonoidHomClass G M N] (g : G) (f : ฮน โ M) (s : Finset ฮน) : g (โ x โ s, f x) = โ x โ s, g (f x) - Finset.sum_induction ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {s : Finset ฮน} {M : Type u_7} [AddCommMonoid M] (f : ฮน โ M) (p : M โ Prop) (hom : โ (a b : M), p a โ p b โ p (a + b)) (addUnit : p 0) (base : โ x โ s, p (f x)) : p (โ x โ s, f x) - Finset.sum_sub_distrib ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {G : Type u_5} {s : Finset ฮน} [SubtractionCommMonoid G] (f g : ฮน โ G) : โ x โ s, (f x - g x) = โ x โ s, f x - โ x โ s, g x - Finset.sum_bijective ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [AddCommMonoid M] {s : Finset ฮน} {t : Finset ฮบ} {f : ฮน โ M} {g : ฮบ โ M} (e : ฮน โ ฮบ) (he : Function.Bijective e) (hst : โ (i : ฮน), i โ s โ e i โ t) (hfg : โ i โ s, f i = g (e i)) : โ i โ s, f i = โ i โ t, g i - ofAdd_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : Multiplicative.ofAdd (โ i โ s, f i) = โ i โ s, Multiplicative.ofAdd (f i) - ofMul_prod ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [CommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : Additive.ofMul (โ i โ s, f i) = โ i โ s, Additive.ofMul (f i) - Equiv.Perm.sum_comp ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (ฯ : Equiv.Perm ฮน) (s : Finset ฮน) (f : ฮน โ M) (hs : {a | ฯ a โ a} โ โs) : โ x โ s, f (ฯ x) = โ x โ s, f x - toAdd_prod ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ Multiplicative M) : Multiplicative.toAdd (โ i โ s, f i) = โ i โ s, Multiplicative.toAdd (f i) - toMul_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [CommMonoid M] (s : Finset ฮน) (f : ฮน โ Additive M) : Additive.toMul (โ i โ s, f i) = โ i โ s, Additive.toMul (f i) - Finset.sum_attach_univ ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] [Fintype ฮน] (f : { i // i โ Finset.univ } โ M) : โ i โ Finset.univ.attach, f i = โ i, f โจi, โฏโฉ - Finset.sum_nbij ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [AddCommMonoid M] {s : Finset ฮน} {t : Finset ฮบ} {f : ฮน โ M} {g : ฮบ โ M} (i : ฮน โ ฮบ) (hi : โ a โ s, i a โ t) (i_inj : Set.InjOn i โs) (i_surj : Set.SurjOn i โs โt) (h : โ a โ s, f a = g (i a)) : โ x โ s, f x = โ x โ t, g x - Equiv.Perm.sum_comp' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] (ฯ : Equiv.Perm ฮน) (s : Finset ฮน) (f : ฮน โ ฮน โ M) (hs : {a | ฯ a โ a} โ โs) : โ x โ s, f (ฯ x) x = โ x โ s, f x ((Equiv.symm ฯ) x) - Finset.sum_equiv ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [AddCommMonoid M] {s : Finset ฮน} {t : Finset ฮบ} {f : ฮน โ M} {g : ฮบ โ M} (e : ฮน โ ฮบ) (hst : โ (i : ฮน), i โ s โ e i โ t) (hfg : โ i โ s, f i = g (e i)) : โ i โ s, f i = โ i โ t, g i - Finset.sum_hom_rel ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} {N : Type u_4} [AddCommMonoid M] [AddCommMonoid N] {r : M โ N โ Prop} {f : ฮน โ M} {g : ฮน โ N} {s : Finset ฮน} (hโ : r 0 0) (hโ : โ (a : ฮน) (b : M) (c : N), r b c โ r (f a + b) (g a + c)) : r (โ x โ s, f x) (โ x โ s, g x) - Finset.sum_mem_multiset ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] [DecidableEq ฮน] (m : Multiset ฮน) (f : { x // x โ m } โ M) (g : ฮน โ M) (hfg : โ (x : { x // x โ m }), f x = g โx) : โ x, f x = โ x โ m.toFinset, g x - Finset.sum_coe_sort_eq_attach ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} (s : Finset ฮน) [AddCommMonoid M] (f : โฅs โ M) : โ i, f i = โ i โ s.attach, f i - Finset.sum_nbij' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [AddCommMonoid M] {s : Finset ฮน} {t : Finset ฮบ} {f : ฮน โ M} {g : ฮบ โ M} (i : ฮน โ ฮบ) (j : ฮบ โ ฮน) (hi : โ a โ s, i a โ t) (hj : โ a โ t, j a โ s) (left_neg : โ a โ s, j (i a) = a) (right_neg : โ a โ t, i (j a) = a) (h : โ a โ s, f a = g (i a)) : โ x โ s, f x = โ x โ t, g x - Finset.sum_bij ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [AddCommMonoid M] {s : Finset ฮน} {t : Finset ฮบ} {f : ฮน โ M} {g : ฮบ โ M} (i : (a : ฮน) โ a โ s โ ฮบ) (hi : โ (a : ฮน) (ha : a โ s), i a ha โ t) (i_inj : โ (aโ : ฮน) (haโ : aโ โ s) (aโ : ฮน) (haโ : aโ โ s), i aโ haโ = i aโ haโ โ aโ = aโ) (i_surj : โ b โ t, โ a, โ (ha : a โ s), i a ha = b) (h : โ (a : ฮน) (ha : a โ s), f a = g (i a ha)) : โ x โ s, f x = โ x โ t, g x - Finset.sum_erase_attach ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {M : Type u_3} [AddCommMonoid M] [DecidableEq ฮน] {s : Finset ฮน} (f : ฮน โ M) (i : โฅs) : โ j โ s.attach.erase i, f โj = โ j โ s.erase โi, f j - Finset.sum_bij' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Defs
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_3} [AddCommMonoid M] {s : Finset ฮน} {t : Finset ฮบ} {f : ฮน โ M} {g : ฮบ โ M} (i : (a : ฮน) โ a โ s โ ฮบ) (j : (a : ฮบ) โ a โ t โ ฮน) (hi : โ (a : ฮน) (ha : a โ s), i a ha โ t) (hj : โ (a : ฮบ) (ha : a โ t), j a ha โ s) (left_neg : โ (a : ฮน) (ha : a โ s), j (i a ha) โฏ = a) (right_neg : โ (a : ฮบ) (ha : a โ t), i (j a ha) โฏ = a) (h : โ (a : ฮน) (ha : a โ s), f a = g (i a ha)) : โ x โ s, f x = โ x โ t, g x - Finset.card_eq_sum_ones ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} (s : Finset ฮน) : s.card = โ x โ s, 1 - Finset.sum_singleton' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] (a : ฮน) : {a}.sum = fun f => f a - Multiset.toFinset_sum_count_eq ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} [DecidableEq ฮน] (s : Multiset ฮน) : โ a โ s.toFinset, Multiset.count a s = s.card - Finset.sum_singleton ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] (f : ฮน โ M) (a : ฮน) : โ x โ {a}, f x = f a - Fintype.sum_subsingleton ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮน : Type u_7} [Fintype ฮน] [AddCommMonoid M] [Subsingleton ฮน] (f : ฮน โ M) (a : ฮน) : โ x, f x = f a - nat_abs_sum_le ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} (s : Finset ฮน) (f : ฮน โ โค) : (โ i โ s, f i).natAbs โค โ i โ s, (f i).natAbs - Finset.sum_range_one ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] (f : โ โ M) : โ k โ Finset.range 1, f k = f 0 - List.sum_toFinset_count_eq_length ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} [DecidableEq ฮน] (l : List ฮน) : โ a โ l.toFinset, List.count a l = l.length - Fintype.sum_unique ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮน : Type u_7} [Fintype ฮน] [AddCommMonoid M] [Unique ฮน] (f : ฮน โ M) : โ x, f x = f default - Finset.nsmul_eq_sum_const ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] (b : M) (n : โ) : n โข b = โ _k โ Finset.range n, b - Finset.sum_unique_nonempty ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [Unique ฮน] (s : Finset ฮน) (f : ฮน โ M) (h : s.Nonempty) : โ x โ s, f x = f default - Finset.card_biUnion_le ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [DecidableEq M] {s : Finset ฮน} {t : ฮน โ Finset M} : (s.biUnion t).card โค โ a โ s, (t a).card - Finset.sum_const ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] (b : M) : โ _x โ s, b = s.card โข b - IsAddUnit.sum_univ_iff ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [Fintype ฮน] [AddCommMonoid M] {f : ฮน โ M} : IsAddUnit (โ a, f a) โ โ (a : ฮน), IsAddUnit (f a) - Fintype.sum_Prop ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] (f : Prop โ M) : โ p, f p = f True + f False - IsAddUnit.sum_iff ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} : IsAddUnit (โ a โ s, f a) โ โ a โ s, IsAddUnit (f a) - Multiset.prod_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮน : Type u_5} [CommMonoid M] (f : ฮน โ Multiset M) (s : Finset ฮน) : (โ x โ s, f x).prod = โ x โ s, (f x).prod - Multiset.sum_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮน : Type u_5} [AddCommMonoid M] (f : ฮน โ Multiset M) (s : Finset ฮน) : (โ x โ s, f x).sum = โ x โ s, (f x).sum - Finset.card_eq_sum_card_image ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [DecidableEq M] (f : ฮน โ M) (s : Finset ฮน) : s.card = โ b โ Finset.image f s, {a โ s | f a = b}.card - Finset.sum_multiset_count ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] [DecidableEq M] (s : Multiset M) : s.sum = โ m โ s.toFinset, Multiset.count m s โข m - Multiset.sum_count_eq_card ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} [DecidableEq ฮน] {s : Finset ฮน} {m : Multiset ฮน} (hms : โ a โ m, a โ s) : โ a โ s, Multiset.count a m = m.card - Finset.sum_const_nat ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {s : Finset ฮน} {m : โ} {f : ฮน โ โ} (hโ : โ x โ s, f x = m) : โ x โ s, f x = s.card * m - Finset.sum_diag ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] (s : Finset ฮน) (f : ฮน ร ฮน โ M) : โ i โ s.diag, f i = โ i โ s, f (i, i) - Finset.card_disjiUnion ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} (s : Finset ฮน) (t : ฮน โ Finset M) (h : (โs).PairwiseDisjoint t) : (s.disjiUnion t h).card = โ a โ s, (t a).card - Finset.card_biUnion ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [DecidableEq M] {t : ฮน โ Finset M} (h : (โs).PairwiseDisjoint t) : (s.biUnion t).card = โ u โ s, (t u).card - Finset.eq_of_card_le_one_of_sum_eq ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {s : Finset ฮน} (hc : s.card โค 1) {f : ฮน โ M} {b : M} (h : โ x โ s, f x = b) (x : ฮน) : x โ s โ f x = b - Finset.sum_congr ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f g : ฮน โ M} (h : sโ = sโ) : (โ x โ sโ, f x = g x) โ sโ.sum f = sโ.sum g - Finset.sum_image ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] {s : Finset ฮบ} {g : ฮบ โ ฮน} : Set.InjOn g โs โ โ x โ Finset.image g s, f x = โ x โ s, f (g x) - Finset.sum_multiset_map_count ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} [DecidableEq ฮน] (s : Multiset ฮน) {M : Type u_5} [AddCommMonoid M] (f : ฮน โ M) : (Multiset.map f s).sum = โ m โ s.toFinset, Multiset.count m s โข f m - Finset.sum_subtype_eq_sum_filter ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] (f : ฮน โ M) {p : ฮน โ Prop} [DecidablePred p] : โ x โ Finset.subtype p s, f โx = โ x โ s with p x, f x - Finset.sum_eq_card_nsmul ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} {b : M} (hf : โ a โ s, f a = b) : โ a โ s, f a = s.card โข b - Finset.sum_multiset_count_of_subset ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] [DecidableEq M] (m : Multiset M) (s : Finset M) (hs : m.toFinset โ s) : m.sum = โ i โ s, Multiset.count i m โข i - List.sum_toFinset ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_5} [DecidableEq ฮน] [AddCommMonoid M] (f : ฮน โ M) {l : List ฮน} (_hl : l.Nodup) : l.toFinset.sum f = (List.map f l).sum - Finset.mem_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {f : ฮน โ Multiset M} (s : Finset ฮน) (b : M) : b โ โ x โ s, f x โ โ a โ s, b โ f a - Multiset.mem_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {a : M} {s : Finset ฮน} {m : ฮน โ Multiset M} : a โ โ i โ s, m i โ โ i โ s, a โ m i - Finset.sum_erase ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] (s : Finset ฮน) {f : ฮน โ M} {a : ฮน} (h : f a = 0) : โ x โ s.erase a, f x = โ x โ s, f x - Finset.sum_set_coe ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {f : ฮน โ M} (s : Set ฮน) [Fintype โs] : โ i, f โi = โ i โ s.toFinset, f i - Finset.prod_pow_eq_pow_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [CommMonoid M] (s : Finset ฮน) (f : ฮน โ โ) (a : M) : โ i โ s, a ^ f i = a ^ โ i โ s, f i - Finset.sum_nsmul_assoc ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ โ) (a : M) : โ i โ s, f i โข a = (โ i โ s, f i) โข a - Finset.sum_subtype_of_mem ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] (f : ฮน โ M) {p : ฮน โ Prop} [DecidablePred p] (h : โ x โ s, p x) : โ x โ Finset.subtype p s, f โx = โ x โ s, f x - Finset.sum_comp_equiv ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮบ โ M} (e : ฮน โ ฮบ) : s.sum (f โ โe) = (Finset.map e.toEmbedding s).sum f - Finset.sum_fiberwise ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮบ] [Fintype ฮบ] (s : Finset ฮน) (g : ฮน โ ฮบ) (f : ฮน โ M) : โ j, โ i โ s with g i = j, f i = โ i โ s, f i - Finset.card_eq_sum_card_fiberwise ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [DecidableEq M] {f : ฮน โ M} {s : Finset ฮน} {t : Finset M} (H : Set.MapsTo f โs โt) : s.card = โ b โ t, {a โ s | f a = b}.card - Finset.sum_fiberwise' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮบ] [Fintype ฮบ] (s : Finset ฮน) (g : ฮน โ ฮบ) (f : ฮบ โ M) : โ j, โ i โ s with g i = j, f j = โ i โ s, f (g i) - Finset.sum_insert_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} {a : ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] (h : f a = 0) : โ x โ insert a s, f x = โ x โ s, f x - Finset.sum_range_succ ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] (f : โ โ M) (n : โ) : โ x โ Finset.range (n + 1), f x = โ x โ Finset.range n, f x + f n - Finset.sum_range_succ_comm ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] (f : โ โ M) (n : โ) : โ x โ Finset.range (n + 1), f x = f n + โ x โ Finset.range n, f x - Finset.sum_subtype ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {p : ฮน โ Prop} {F : Fintype (Subtype p)} (s : Finset ฮน) (h : โ (x : ฮน), x โ s โ p x) (f : ฮน โ M) : โ a โ s, f a = โ a, f โa - Finset.eventually_constant_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] {u : โ โ M} {N : โ} (hu : โ n โฅ N, u n = 0) {n : โ} (hn : N โค n) : โ k โ Finset.range n, u k = โ k โ Finset.range N, u k - Finset.sum_card_fiberwise_eq_card_filter ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_5} [DecidableEq ฮบ] (s : Finset ฮน) (t : Finset ฮบ) (g : ฮน โ ฮบ) : โ j โ t, {i โ s | g i = j}.card = {i โ s | g i โ t}.card - Finset.sum_cons' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} {a : ฮน} [AddCommMonoid M] (h : a โ s) : (Finset.cons a s h).sum = fun f => f a + โ x โ s, f x - Multiset.toFinset_sum_count_nsmul_eq ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} [DecidableEq ฮน] (s : Multiset ฮน) : โ a โ s.toFinset, Multiset.count a s โข {a} = s - Finset.sum_cons ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} {a : ฮน} [AddCommMonoid M] {f : ฮน โ M} (h : a โ s) : โ x โ Finset.cons a s h, f x = f a + โ x โ s, f x - Finset.sum_extend_by_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] (s : Finset ฮน) (f : ฮน โ M) : (โ i โ s, if i โ s then f i else 0) = โ i โ s, f i - Finset.sum_filter ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] (p : ฮน โ Prop) [DecidablePred p] (f : ฮน โ M) : โ a โ s with p a, f a = โ a โ s, if p a then f a else 0 - Finset.sum_map_equiv ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} (e : ฮน โ ฮบ) : (Finset.map e.toEmbedding s).sum (f โ โe.symm) = s.sum f - Finset.sum_pair ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] {a b : ฮน} (h : a โ b) : โ x โ {a, b}, f x = f a + f b - Fintype.sum_subset ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮน : Type u_7} [Fintype ฮน] [AddCommMonoid M] {s : Finset ฮน} {f : ฮน โ M} (h : โ (i : ฮน), f i โ 0 โ i โ s) : โ i โ s, f i = โ i, f i - Finset.add_sum_erase ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] (s : Finset ฮน) (f : ฮน โ M) {a : ฮน} (h : a โ s) : f a + โ x โ s.erase a, f x = โ x โ s, f x - Finset.sum_disjiUnion ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] {f : ฮน โ M} (s : Finset ฮบ) (t : ฮบ โ Finset ฮน) (h : (โs).PairwiseDisjoint t) : โ x โ s.disjiUnion t h, f x = โ i โ s, โ x โ t i, f x - Finset.sum_erase_add ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] (s : Finset ฮน) (f : ฮน โ M) {a : ฮน} (h : a โ s) : โ x โ s.erase a, f x + f a = โ x โ s, f x - Finset.sum_flip ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] {n : โ} (f : โ โ M) : โ r โ Finset.range (n + 1), f (n - r) = โ k โ Finset.range (n + 1), f k - Finset.sum_attach ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : โ x โ s.attach, f โx = โ x โ s, f x - Finset.sum_eq_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} (h : โ x โ s, f x = 0) : โ x โ s, f x = 0 - Finset.sum_list_count ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] [DecidableEq M] (s : List M) : s.sum = โ m โ s.toFinset, List.count m s โข m - Finset.sum_biUnion ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] {s : Finset ฮบ} {t : ฮบ โ Finset ฮน} (hs : (โs).PairwiseDisjoint t) : โ x โ s.biUnion t, f x = โ x โ s, โ i โ t x, f i - Finset.sum_eq_single_of_mem ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {s : Finset ฮน} {f : ฮน โ M} (a : ฮน) (h : a โ s) (hโ : โ b โ s, b โ a โ f b = 0) : โ x โ s, f x = f a - Finset.sum_erase_eq_sub ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {G : Type u_3} {s : Finset ฮน} [AddCommGroup G] [DecidableEq ฮน] {f : ฮน โ G} {a : ฮน} (h : a โ s) : โ x โ s.erase a, f x = โ x โ s, f x - f a - Finset.exists_ne_zero_of_sum_ne_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} (h : โ x โ s, f x โ 0) : โ a โ s, f a โ 0 - Finset.sum_insert' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} {a : ฮน} [AddCommMonoid M] [DecidableEq ฮน] (h : a โ s) : (insert a s).sum = fun f => f a + โ x โ s, f x - Finset.sum_insert ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} {a : ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] : a โ s โ โ x โ insert a s, f x = f a + โ x โ s, f x - Finset.sum_disjUnion ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} (h : Disjoint sโ sโ) : โ x โ sโ.disjUnion sโ h, f x = โ x โ sโ, f x + โ x โ sโ, f x - Finset.sum_insert_of_eq_zero_if_notMem ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} {a : ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] (h : a โ s โ f a = 0) : โ x โ insert a s, f x = โ x โ s, f x - Finset.sum_insert_of_eq_zero_if_not_mem ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} {a : ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] (h : a โ s โ f a = 0) : โ x โ insert a s, f x = โ x โ s, f x - Finset.sum_add_sum_compl ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [Fintype ฮน] [DecidableEq ฮน] (s : Finset ฮน) (f : ฮน โ M) : โ i โ s, f i + โ i โ sแถ, f i = โ i, f i - Finset.sum_comp ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] [DecidableEq ฮบ] (f : ฮบ โ M) (g : ฮน โ ฮบ) : โ a โ s, f (g a) = โ b โ Finset.image g s, {a โ s | g a = b}.card โข f b - Finset.sum_compl_add_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [Fintype ฮน] [DecidableEq ฮน] (s : Finset ฮน) (f : ฮน โ M) : โ i โ sแถ, f i + โ i โ s, f i = โ i, f i - Finset.sum_insert_sub ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {G : Type u_3} {s : Finset ฮน} {a : ฮน} [AddCommGroup G] [DecidableEq ฮน] (ha : a โ s) (f : ฮน โ G) : โ x โ insert a s, f x - f a = โ x โ s, f x - IsCompl.sum_add_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [Fintype ฮน] {s t : Finset ฮน} (h : IsCompl s t) (f : ฮน โ M) : โ i โ s, f i + โ i โ t, f i = โ i, f i - Finset.sum_eq_zero_iff ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} [Subsingleton (AddUnits M)] : โ i โ s, f i = 0 โ โ i โ s, f i = 0 - Finset.sum_filter_of_ne ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} {p : ฮน โ Prop} [DecidablePred p] (hp : โ x โ s, f x โ 0 โ p x) : โ x โ s with p x, f x = โ x โ s, f x - Finset.sum_ite_mem_eq ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [Fintype ฮน] (s : Finset ฮน) (f : ฮน โ M) [DecidablePred fun x => x โ s] : (โ i, if i โ s then f i else 0) = โ i โ s, f i - Finset.sum_list_map_count ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] (l : List ฮน) (f : ฮน โ M) : (List.map f l).sum = โ m โ l.toFinset, List.count m l โข f m - Finset.sum_range_add ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] (f : โ โ M) (n m : โ) : โ x โ Finset.range (n + m), f x = โ x โ Finset.range n, f x + โ x โ Finset.range m, f (n + x) - Finset.sum_range_sub ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{G : Type u_3} [AddCommGroup G] (f : โ โ G) (n : โ) : โ i โ Finset.range n, (f (i + 1) - f i) = f n - f 0 - Finset.sum_range_sub' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{G : Type u_3} [AddCommGroup G] (f : โ โ G) (n : โ) : โ i โ Finset.range n, (f i - f (i + 1)) = f 0 - f n - Finset.sum_sdiff ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] (h : sโ โ sโ) : โ x โ sโ \ sโ, f x + โ x โ sโ, f x = โ x โ sโ, f x - Finset.sum_sumElim ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] (s : Finset ฮน) (t : Finset ฮบ) (f : ฮน โ M) (g : ฮบ โ M) : โ x โ s.disjSum t, Sum.elim f g x = โ x โ s, f x + โ x โ t, g x - Finset.sum_add_distrib ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f g : ฮน โ M} : โ x โ s, (f x + g x) = โ x โ s, f x + โ x โ s, g x - Finset.sum_disjSum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] (s : Finset ฮน) (t : Finset ฮบ) (f : ฮน โ ฮบ โ M) : โ x โ s.disjSum t, f x = โ x โ s, f (Sum.inl x) + โ x โ t, f (Sum.inr x) - Finset.sum_disj_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] (s : Finset ฮน) (t : Finset ฮบ) (f : ฮน โ ฮบ โ M) : โ x โ s.disjSum t, f x = โ x โ s, f (Sum.inl x) + โ x โ t, f (Sum.inr x) - Finset.sum_filter_ne_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {f : ฮน โ M} (s : Finset ฮน) [(x : ฮน) โ Decidable (f x โ 0)] : โ x โ s with f x โ 0, f x = โ x โ s, f x - Finset.sum_list_count_of_subset ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] [DecidableEq M] (m : List M) (s : Finset M) (hs : m.toFinset โ s) : m.sum = โ i โ s, List.count i m โข i - Finset.sum_union ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] (h : Disjoint sโ sโ) : โ x โ sโ โช sโ, f x = โ x โ sโ, f x + โ x โ sโ, f x - Finset.sum_eq_fold ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] (s : Finset ฮน) (f : ฮน โ M) : โ i โ s, f i = Finset.fold (fun x1 x2 => x1 + x2) 0 f s - Finset.sum_fiberwise_of_maps_to ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] {s : Finset ฮน} {t : Finset ฮบ} [DecidableEq ฮบ] {g : ฮน โ ฮบ} (h : โ i โ s, g i โ t) (f : ฮน โ M) : โ j โ t, โ i โ s with g i = j, f i = โ i โ s, f i - Finset.sum_sum_eq_sum_toLeft_add_sum_toRight ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] (s : Finset (ฮน โ ฮบ)) (f : ฮน โ ฮบ โ M) : โ x โ s, f x = โ x โ s.toLeft, f (Sum.inl x) + โ x โ s.toRight, f (Sum.inr x) - Finset.sum_fiberwise_eq_sum_filter ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮบ] (s : Finset ฮน) (t : Finset ฮบ) (g : ฮน โ ฮบ) (f : ฮน โ M) : โ j โ t, โ i โ s with g i = j, f i = โ i โ s with g i โ t, f i - Finset.sum_fiberwise_of_maps_to' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] {s : Finset ฮน} {t : Finset ฮบ} [DecidableEq ฮบ] {g : ฮน โ ฮบ} (h : โ i โ s, g i โ t) (f : ฮบ โ M) : โ j โ t, โ i โ s with g i = j, f j = โ i โ s, f (g i) - Finset.sum_finset_coe ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] (f : ฮน โ M) (s : Finset ฮน) : โ i, f โi = โ i โ s, f i - Finset.sum_range_add_sub_sum_range ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{G : Type u_3} [AddCommGroup G] (f : โ โ G) (n m : โ) : โ k โ Finset.range (n + m), f k - โ k โ Finset.range n, f k = โ k โ Finset.range m, f (n + k) - Finset.sum_range_succ' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] (f : โ โ M) (n : โ) : โ k โ Finset.range (n + 1), f k = โ k โ Finset.range n, f (k + 1) + f 0 - Finset.sum_sdiff_eq_sub ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {G : Type u_3} {sโ sโ : Finset ฮน} [AddCommGroup G] [DecidableEq ฮน] {f : ฮน โ G} (h : sโ โ sโ) : โ x โ sโ \ sโ, f x = โ x โ sโ, f x - โ x โ sโ, f x - Finset.sum_sdiff_eq_sum_sdiff_iff ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [DecidableEq ฮน] [AddCancelCommMonoid M] {s t : Finset ฮน} {f : ฮน โ M} : โ i โ s \ t, f i = โ i โ t \ s, f i โ โ i โ s, f i = โ i โ t, f i - Finset.sum_sdiff_ne_sum_sdiff_iff ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [DecidableEq ฮน] [AddCancelCommMonoid M] {s t : Finset ฮน} {f : ฮน โ M} : โ i โ s \ t, f i โ โ i โ t \ s, f i โ โ i โ s, f i โ โ i โ t, f i - Finset.sum_subset ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} (h : sโ โ sโ) (hf : โ x โ sโ, x โ sโ โ f x = 0) : โ x โ sโ, f x = โ x โ sโ, f x - Finset.sum_fiberwise_eq_sum_filter' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮบ] (s : Finset ฮน) (t : Finset ฮบ) (g : ฮน โ ฮบ) (f : ฮบ โ M) : โ j โ t, โ i โ s with g i = j, f j = โ i โ s with g i โ t, f (g i) - Finset.sum_filter_add_sum_filter_not ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] (s : Finset ฮน) (p : ฮน โ Prop) [DecidablePred p] [(x : ฮน) โ Decidable ยฌp x] (f : ฮน โ M) : โ x โ s with p x, f x + โ x โ s with ยฌp x, f x = โ x โ s, f x - Finset.sum_filter_not_add_sum_filter ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] (s : Finset ฮน) (p : ฮน โ Prop) [DecidablePred p] [(x : ฮน) โ Decidable ยฌp x] (f : ฮน โ M) : โ x โ s with ยฌp x, f x + โ x โ s with p x, f x = โ x โ s, f x - Finset.eq_sum_range_sub ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{G : Type u_3} [AddCommGroup G] (f : โ โ G) (n : โ) : f n = f 0 + โ i โ Finset.range n, (f (i + 1) - f i) - Finset.sum_image_of_pairwise_eq_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] {f : ฮบ โ ฮน} {g : ฮน โ M} {I : Finset ฮบ} (hf : (โI).Pairwise fun i j => f i = f j โ g (f i) = 0) : โ s โ Finset.image f I, g s = โ i โ I, g (f i) - Finset.sum_union_eq_left ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] (hs : โ a โ sโ, a โ sโ โ f a = 0) : โ a โ sโ โช sโ, f a = โ a โ sโ, f a - Finset.sum_union_eq_right ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] (hs : โ a โ sโ, a โ sโ โ f a = 0) : โ a โ sโ โช sโ, f a = โ a โ sโ, f a - Finset.card_nsmul_add_sum ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} {b : M} : s.card โข b + โ a โ s, f a = โ a โ s, (b + f a) - Finset.sum_add_card_nsmul ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} {b : M} : โ a โ s, f a + s.card โข b = โ a โ s, (f a + b) - Finset.sum_erase_lt_of_pos ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_5} [DecidableEq ฮน] [AddCommMonoid ฮบ] [LT ฮบ] [AddLeftStrictMono ฮบ] {s : Finset ฮน} {d : ฮน} (hd : d โ s) {f : ฮน โ ฮบ} (hdf : 0 < f d) : โ m โ s.erase d, f m < โ m โ s, f m - Finset.sum_image' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] {s : Finset ฮบ} {g : ฮบ โ ฮน} (h : ฮบ โ M) (eq : โ i โ s, f (g i) = โ j โ s with g j = g i, h j) : โ a โ Finset.image g s, f a = โ i โ s, h i - Finset.sum_eq_single ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {s : Finset ฮน} {f : ฮน โ M} (a : ฮน) (hโ : โ b โ s, b โ a โ f b = 0) (hโ : a โ s โ f a = 0) : โ x โ s, f x = f a - Fintype.sum_fiberwise' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮบ : Type u_6} {ฮน : Type u_7} [Fintype ฮน] [Fintype ฮบ] [AddCommMonoid M] [DecidableEq ฮบ] (g : ฮน โ ฮบ) (f : ฮบ โ M) : โ j, โ _i, f j = โ i, f (g i) - Fintype.sum_of_injective ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮบ : Type u_6} {ฮน : Type u_7} [Fintype ฮน] [Fintype ฮบ] [AddCommMonoid M] (e : ฮน โ ฮบ) (he : Function.Injective e) (f : ฮน โ M) (g : ฮบ โ M) (h' : โ i โ Set.range e, g i = 0) (h : โ (i : ฮน), f i = g (e i)) : โ i, f i = โ j, g j - Finset.eq_sum_range_sub' ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{G : Type u_3} [AddCommGroup G] (f : โ โ G) (n : โ) : f n = โ i โ Finset.range (n + 1), if i = 0 then f 0 else f i - f (i - 1) - Finset.sum_eq_ite ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] {s : Finset ฮน} {f : ฮน โ M} (a : ฮน) (hโ : โ b โ s, b โ a โ f b = 0) : โ x โ s, f x = if a โ s then f a else 0 - Finset.sum_range_induction ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} [AddCommMonoid M] (f s : โ โ M) (base : s 0 = 0) (n : โ) (step : โ k < n, s (k + 1) = s k + f k) : โ k โ Finset.range n, f k = s n - Finset.sum_cancels_of_partition_cancels ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} (R : Setoid ฮน) [DecidableRel โR] (h : โ x โ s, โ a โ s with R a x, f a = 0) : โ x โ s, f x = 0 - Finset.sum_image_of_disjoint ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] [PartialOrder ฮน] [OrderBot ฮน] {f : ฮบ โ ฮน} {g : ฮน โ M} (hg_bot : g โฅ = 0) {I : Finset ฮบ} (hf_disj : (โI).PairwiseDisjoint f) : โ s โ Finset.image f I, g s = โ i โ I, g (f i) - Finset.sum_partition ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} (R : Setoid ฮน) [DecidableRel โR] : โ x โ s, f x = โ xbar โ Finset.image (Quotient.mk R) s, โ y โ s with โฆyโง = xbar, f y - Finset.sum_coe_sort ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} (s : Finset ฮน) [AddCommMonoid M] (f : ฮน โ M) : โ i, f โi = โ i โ s, f i - Finset.sum_filter_of_pairwise_eq_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {ฮบ : Type u_2} {M : Type u_4} [AddCommMonoid M] [DecidableEq ฮน] {f : ฮบ โ ฮน} {g : ฮน โ M} {n : ฮบ} {I : Finset ฮบ} (hn : n โ I) (hf : (โI).Pairwise fun i j => f i = f j โ g (f i) = 0) : โ j โ I with f j = f n, g (f j) = g (f n) - Fintype.sum_fiberwise ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮบ : Type u_6} {ฮน : Type u_7} [Fintype ฮน] [Fintype ฮบ] [AddCommMonoid M] [DecidableEq ฮบ] (g : ฮน โ ฮบ) (f : ฮน โ M) : โ j, โ i, f โi = โ i, f i - Finset.sum_subset_zero_on_sdiff ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f g : ฮน โ M} [DecidableEq ฮน] (h : sโ โ sโ) (hg : โ x โ sโ \ sโ, g x = 0) (hfg : โ x โ sโ, f x = g x) : โ i โ sโ, f i = โ i โ sโ, g i - Finset.sum_union_inter ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {sโ sโ : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} [DecidableEq ฮน] : โ x โ sโ โช sโ, f x + โ x โ sโ โฉ sโ, f x = โ x โ sโ, f x + โ x โ sโ, f x - Finset.eq_zero_of_sum_eq_zero ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {s : Finset ฮน} {f : ฮน โ M} {a : ฮน} (hp : โ x โ s, f x = 0) (h1 : โ x โ s, x โ a โ f x = 0) (x : ฮน) : x โ s โ f x = 0 - Finset.sum_sdiff_sub_sum_sdiff ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {G : Type u_3} {sโ sโ : Finset ฮน} [AddCommGroup G] [DecidableEq ฮน] {f : ฮน โ G} : โ x โ sโ \ sโ, f x - โ x โ sโ \ sโ, f x = โ x โ sโ, f x - โ x โ sโ, f x - Finset.sum_subtype_map_embedding ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {p : ฮน โ Prop} {s : Finset { x // p x }} {f : { x // p x } โ M} {g : ฮน โ M} (h : โ x โ s, g โx = f x) : โ x โ Finset.map (Function.Embedding.subtype fun x => p x) s, g x = โ x โ s, f x - Finset.sum_eq_add_of_mem ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {s : Finset ฮน} {f : ฮน โ M} (a b : ฮน) (ha : a โ s) (hb : b โ s) (hn : a โ b) (hโ : โ c โ s, c โ a โง c โ b โ f c = 0) : โ x โ s, f x = f a + f b - Finset.sum_add_eq_sum_add_of_exists ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] {s : Finset ฮน} {f : ฮน โ M} {bโ bโ : M} (a : ฮน) (ha : a โ s) (h : f a + bโ = f a + bโ) : โ a โ s, f a + bโ = โ a โ s, f a + bโ - Finset.sum_ninvolution ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} {s : Finset ฮน} [AddCommMonoid M] {f : ฮน โ M} (g : ฮน โ ฮน) (hgโ : โ (a : ฮน), f a + f (g a) = 0) (hgโ : โ (a : ฮน), f a โ 0 โ g a โ a) (g_mem : โ (a : ฮน), g a โ s) (hgโ : โ (a : ฮน), g (g a) = a) : โ x โ s, f x = 0 - Fintype.sum_subtype_add_sum_subtype ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{M : Type u_4} {ฮน : Type u_7} [Fintype ฮน] [AddCommMonoid M] (p : ฮน โ Prop) (f : ฮน โ M) [DecidablePred p] : โ i, f โi + โ i, f โi = โ i, f i - Finset.sum_congr_set ๐ Mathlib.Algebra.BigOperators.Group.Finset.Basic
{ฮน : Type u_1} {M : Type u_4} [AddCommMonoid M] [Fintype ฮน] (s : Set ฮน) [DecidablePred fun x => x โ s] (f : ฮน โ M) (g : โs โ M) (w : โ (x : ฮน) (hx : x โ s), f x = g โจx, hxโฉ) (w' : โ x โ s, f x = 0) : โ i, f i = โ i, g i
About
Loogle searches Lean and Mathlib definitions and theorems.
You can use Loogle from within the Lean4 VSCode language extension
using (by default) Ctrl-K Ctrl-S. You can also try the
#loogle command from LeanSearchClient,
the CLI version, the Loogle
VS Code extension, the lean.nvim
integration or the Zulip bot.
Usage
Loogle finds definitions and lemmas in various ways:
By constant:
๐Real.sin
finds all lemmas whose statement somehow mentions the sine function.By lemma name substring:
๐"differ"
finds all lemmas that have"differ"somewhere in their lemma name.By subexpression:
๐_ * (_ ^ _)
finds all lemmas whose statements somewhere include a product where the second argument is raised to some power.The pattern can also be non-linear, as in
๐Real.sqrt ?a * Real.sqrt ?aIf the pattern has parameters, they are matched in any order. Both of these will find
List.map:
๐(?a -> ?b) -> List ?a -> List ?b
๐List ?a -> (?a -> ?b) -> List ?bBy main conclusion:
๐|- tsum _ = _ * tsum _
finds all lemmas where the conclusion (the subexpression to the right of allโandโ) has the given shape.As before, if the pattern has parameters, they are matched against the hypotheses of the lemma in any order; for example,
๐|- _ < _ โ tsum _ < tsum _
will findtsum_lt_tsumeven though the hypothesisf i < g iis not the last.
If you pass more than one such search filter, separated by commas
Loogle will return lemmas which match all of them. The
search
๐ Real.sin, "two", tsum, _ * _, _ ^ _, |- _ < _ โ _
would find all lemmas which mention the constants Real.sin
and tsum, have "two" as a substring of the
lemma name, include a product and a power somewhere in the type,
and have a hypothesis of the form _ < _ (if
there were any such lemmas). Metavariables (?a) are
assigned independently in each filter.
The #lucky button will directly send you to the
documentation of the first hit.
Source code
You can find the source code for this service at https://github.com/nomeata/loogle. The https://loogle.lean-lang.org/ service is provided by the Lean FRO.
This is Loogle revision 0ac13cd serving mathlib revision a7f816c