src/HOL/Analysis/Set_Integral.thy
changeset 82969 dedd9d13c79c
parent 81184 f270cd6ee185
child 83011 d35875d530a2
equal deleted inserted replaced
82968:b2b88d5b01b6 82969:dedd9d13c79c
   606 syntax_consts
   606 syntax_consts
   607   "_ascii_complex_set_lebesgue_integral" == complex_set_lebesgue_integral
   607   "_ascii_complex_set_lebesgue_integral" == complex_set_lebesgue_integral
   608 translations
   608 translations
   609   "CLINT x:A|M. f" == "CONST complex_set_lebesgue_integral M A (\<lambda>x. f)"
   609   "CLINT x:A|M. f" == "CONST complex_set_lebesgue_integral M A (\<lambda>x. f)"
   610 
   610 
   611 lemma set_measurable_continuous_on_ivl:
   611 lemma set_measurable_continuous_on:
   612   assumes "continuous_on {a..b} (f :: real \<Rightarrow> real)"
   612   fixes f g :: "'a::topological_space \<Rightarrow> 'b::real_normed_vector"
   613   shows "set_borel_measurable borel {a..b} f"
   613   shows "A \<in> sets borel \<Longrightarrow> continuous_on A f \<Longrightarrow> set_borel_measurable borel A f"
   614   unfolding set_borel_measurable_def
   614   by (meson borel_measurable_continuous_on_indicator
   615   by (rule borel_measurable_continuous_on_indicator[OF _ assms]) simp
   615       set_borel_measurable_def)
   616 
   616 
   617 section \<open>NN Set Integrals\<close>
   617 section \<open>NN Set Integrals\<close>
   618 
   618 
   619 text\<open>This notation is from Sébastien Gouëzel: His use is not directly in line with the
   619 text\<open>This notation is from Sébastien Gouëzel: His use is not directly in line with the
   620 notations in this file, they are more in line with sum, and more readable he thinks.\<close>
   620 notations in this file, they are more in line with sum, and more readable he thinks.\<close>