src/HOL/Analysis/Linear_Algebra.thy
changeset 69510 0f31dd2e540d
parent 68901 4824cc40f42e
child 69513 42e08052dae8
--- a/src/HOL/Analysis/Linear_Algebra.thy	Thu Dec 27 19:48:41 2018 +0100
+++ b/src/HOL/Analysis/Linear_Algebra.thy	Thu Dec 27 21:00:50 2018 +0100
@@ -106,12 +106,6 @@
   using sum_norm_le[OF K] sum_constant[symmetric]
   by simp
 
-lemma sum_group:
-  assumes fS: "finite S" and fT: "finite T" and fST: "f ` S \<subseteq> T"
-  shows "sum (\<lambda>y. sum g {x. x \<in> S \<and> f x = y}) T = sum g S"
-  unfolding sum_image_gen[OF fS, of g f]
-  by (auto intro: sum.neutral sum.mono_neutral_right[OF fT fST])
-
 lemma vector_eq_ldot: "(\<forall>x. x \<bullet> y = x \<bullet> z) \<longleftrightarrow> y = z"
 proof
   assume "\<forall>x. x \<bullet> y = x \<bullet> z"