src/HOL/Analysis/Linear_Algebra.thy
changeset 66804 3f9bb52082c4
parent 66641 ff2e0115fea4
child 67399 eab6ce8368fa
equal deleted inserted replaced
66803:dd8922885a68 66804:3f9bb52082c4
  1884   shows "(\<Sum>x\<in>P. norm (f x)) \<le> 2 * real DIM('n) * e"
  1884   shows "(\<Sum>x\<in>P. norm (f x)) \<le> 2 * real DIM('n) * e"
  1885 proof -
  1885 proof -
  1886   have "(\<Sum>x\<in>P. norm (f x)) \<le> (\<Sum>x\<in>P. \<Sum>b\<in>Basis. \<bar>f x \<bullet> b\<bar>)"
  1886   have "(\<Sum>x\<in>P. norm (f x)) \<le> (\<Sum>x\<in>P. \<Sum>b\<in>Basis. \<bar>f x \<bullet> b\<bar>)"
  1887     by (rule sum_mono) (rule norm_le_l1)
  1887     by (rule sum_mono) (rule norm_le_l1)
  1888   also have "(\<Sum>x\<in>P. \<Sum>b\<in>Basis. \<bar>f x \<bullet> b\<bar>) = (\<Sum>b\<in>Basis. \<Sum>x\<in>P. \<bar>f x \<bullet> b\<bar>)"
  1888   also have "(\<Sum>x\<in>P. \<Sum>b\<in>Basis. \<bar>f x \<bullet> b\<bar>) = (\<Sum>b\<in>Basis. \<Sum>x\<in>P. \<bar>f x \<bullet> b\<bar>)"
  1889     by (rule sum.commute)
  1889     by (rule sum.swap)
  1890   also have "\<dots> \<le> of_nat (card (Basis :: 'n set)) * (2 * e)"
  1890   also have "\<dots> \<le> of_nat (card (Basis :: 'n set)) * (2 * e)"
  1891   proof (rule sum_bounded_above)
  1891   proof (rule sum_bounded_above)
  1892     fix i :: 'n
  1892     fix i :: 'n
  1893     assume i: "i \<in> Basis"
  1893     assume i: "i \<in> Basis"
  1894     have "norm (\<Sum>x\<in>P. \<bar>f x \<bullet> i\<bar>) \<le>
  1894     have "norm (\<Sum>x\<in>P. \<bar>f x \<bullet> i\<bar>) \<le>