src/HOL/Analysis/Equivalence_Lebesgue_Henstock_Integration.thy
changeset 70726 91587befabfd
parent 70721 47258727fa42
child 70802 160eaf566bcb
equal deleted inserted replaced
70725:e19c18b4a0dd 70726:91587befabfd
  4842     by (rule absolutely_integrable_spike) (auto intro: empty_imp_negligible)
  4842     by (rule absolutely_integrable_spike) (auto intro: empty_imp_negligible)
  4843   then show ?thesis
  4843   then show ?thesis
  4844     unfolding absolutely_integrable_restrict_UNIV .
  4844     unfolding absolutely_integrable_restrict_UNIV .
  4845 qed
  4845 qed
  4846 
  4846 
       
  4847 lemma absolutely_integrable_on_combine:
       
  4848   fixes f :: "real \<Rightarrow> 'a::euclidean_space"
       
  4849   assumes "f absolutely_integrable_on {a..c}"
       
  4850     and "f absolutely_integrable_on {c..b}"
       
  4851     and "a \<le> c"
       
  4852     and "c \<le> b"
       
  4853   shows "f absolutely_integrable_on {a..b}"
       
  4854   by (metis absolutely_integrable_Un assms ivl_disj_un_two_touch(4))
       
  4855 
  4847 lemma uniform_limit_set_lebesgue_integral_at_top:
  4856 lemma uniform_limit_set_lebesgue_integral_at_top:
  4848   fixes f :: "'a \<Rightarrow> real \<Rightarrow> 'b::{banach, second_countable_topology}"
  4857   fixes f :: "'a \<Rightarrow> real \<Rightarrow> 'b::{banach, second_countable_topology}"
  4849     and g :: "real \<Rightarrow> real"
  4858     and g :: "real \<Rightarrow> real"
  4850   assumes bound: "\<And>x y. x \<in> A \<Longrightarrow> y \<ge> a \<Longrightarrow> norm (f x y) \<le> g y"
  4859   assumes bound: "\<And>x y. x \<in> A \<Longrightarrow> y \<ge> a \<Longrightarrow> norm (f x y) \<le> g y"
  4851   assumes integrable: "set_integrable M {a..} g"
  4860   assumes integrable: "set_integrable M {a..} g"