src/HOL/Analysis/Improper_Integral.thy
changeset 66552 507a42c0a0ff
parent 66497 18a6478a574c
child 67399 eab6ce8368fa
equal deleted inserted replaced
66540:1f955cdd9e59 66552:507a42c0a0ff
   218         using \<gamma> [OF \<open>f \<in> F\<close> tag' fine'] integral_reflect
   218         using \<gamma> [OF \<open>f \<in> F\<close> tag' fine'] integral_reflect
   219         by (metis (mono_tags, lifting) Henstock_Kurzweil_Integration.integral_cong comp_apply split_def sum.cong)
   219         by (metis (mono_tags, lifting) Henstock_Kurzweil_Integration.integral_cong comp_apply split_def sum.cong)
   220     qed
   220     qed
   221   qed
   221   qed
   222   then show ?thesis
   222   then show ?thesis
   223     using assms by (auto simp: equiintegrable_on_def integrable_eq)
   223     using assms
       
   224     apply (auto simp: equiintegrable_on_def)
       
   225     apply (rule integrable_eq)
       
   226     by auto 
   224 qed
   227 qed
   225 
   228 
   226 subsection\<open>Subinterval restrictions for equiintegrable families\<close>
   229 subsection\<open>Subinterval restrictions for equiintegrable families\<close>
   227 
   230 
   228 text\<open>First, some technical lemmas about minimizing a "flat" part of a sum over a division.\<close>
   231 text\<open>First, some technical lemmas about minimizing a "flat" part of a sum over a division.\<close>