src/HOL/Analysis/Linear_Algebra.thy
changeset 63918 6bf55e6e0b75
parent 63886 685fb01256af
child 63938 f6ce08859d4c
--- a/src/HOL/Analysis/Linear_Algebra.thy	Mon Sep 19 12:53:30 2016 +0200
+++ b/src/HOL/Analysis/Linear_Algebra.thy	Mon Sep 19 20:06:21 2016 +0200
@@ -1960,7 +1960,7 @@
     qed
     from setsum_norm_le[of _ ?g, OF th]
     show "norm (f x) \<le> ?B * norm x"
-      unfolding th0 setsum_left_distrib by metis
+      unfolding th0 setsum_distrib_right by metis
   qed
 qed
 
@@ -2021,7 +2021,7 @@
     unfolding bilinear_setsum[OF bh finite_Basis finite_Basis] ..
   finally have th: "norm (h x y) = \<dots>" .
   show "norm (h x y) \<le> (\<Sum>i\<in>Basis. \<Sum>j\<in>Basis. norm (h i j)) * norm x * norm y"
-    apply (auto simp add: setsum_left_distrib th setsum.cartesian_product)
+    apply (auto simp add: setsum_distrib_right th setsum.cartesian_product)
     apply (rule setsum_norm_le)
     apply simp
     apply (auto simp add: bilinear_rmul[OF bh] bilinear_lmul[OF bh]