src/HOL/Analysis/Henstock_Kurzweil_Integration.thy
changeset 72548 16345c07bd8c
parent 72445 2c2de074832e
child 72569 d56e4eeae967
equal deleted inserted replaced
72539:97f12d2c8bf2 72548:16345c07bd8c
  5797       if inp: "(x, l) \<in> p" "(y, m) \<in> p" and ne: "(x, l) \<noteq> (y, m)" and "l = m" for x l y m
  5797       if inp: "(x, l) \<in> p" "(y, m) \<in> p" and ne: "(x, l) \<noteq> (y, m)" and "l = m" for x l y m
  5798     proof -
  5798     proof -
  5799       obtain u v where uv: "l = cbox u v"
  5799       obtain u v where uv: "l = cbox u v"
  5800         using inp p'(4) by blast
  5800         using inp p'(4) by blast
  5801       have "content (cbox u v) = 0"
  5801       have "content (cbox u v) = 0"
  5802         unfolding content_eq_0_interior using that p(1) uv by auto
  5802         unfolding content_eq_0_interior using that p(1) uv
       
  5803         by (auto dest: tagged_partial_division_ofD)
  5803       then show ?thesis
  5804       then show ?thesis
  5804         using uv by blast
  5805         using uv by blast
  5805     qed
  5806     qed
  5806     then have "(\<Sum>(x, K)\<in>p. integral K f) = (\<Sum>K\<in>snd ` p. integral K f)"
  5807     then have "(\<Sum>(x, K)\<in>p. integral K f) = (\<Sum>K\<in>snd ` p. integral K f)"
  5807       apply (subst sum.reindex_nontrivial [OF \<open>finite p\<close>])
  5808       apply (subst sum.reindex_nontrivial [OF \<open>finite p\<close>])
  5822     and tag: "p tagged_partial_division_of (cbox a b)"
  5823     and tag: "p tagged_partial_division_of (cbox a b)"
  5823     and "d fine p"
  5824     and "d fine p"
  5824   shows "sum (\<lambda>(x,k). norm (content k *\<^sub>R f x - integral k f)) p \<le> 2 * real (DIM('n)) * e"
  5825   shows "sum (\<lambda>(x,k). norm (content k *\<^sub>R f x - integral k f)) p \<le> 2 * real (DIM('n)) * e"
  5825 proof -
  5826 proof -
  5826   have "finite p"
  5827   have "finite p"
  5827     using tag by blast
  5828     using tag tagged_partial_division_ofD by blast
  5828   then show ?thesis
  5829   then show ?thesis
  5829     unfolding split_def
  5830     unfolding split_def
  5830   proof (rule sum_norm_allsubsets_bound)
  5831   proof (rule sum_norm_allsubsets_bound)
  5831     fix Q
  5832     fix Q
  5832     assume Q: "Q \<subseteq> p"
  5833     assume Q: "Q \<subseteq> p"