src/HOL/Analysis/Set_Integral.thy
changeset 82969 dedd9d13c79c
parent 81184 f270cd6ee185
child 83011 d35875d530a2
--- a/src/HOL/Analysis/Set_Integral.thy	Thu Aug 07 22:42:21 2025 +0200
+++ b/src/HOL/Analysis/Set_Integral.thy	Fri Aug 08 16:46:03 2025 +0100
@@ -608,11 +608,11 @@
 translations
   "CLINT x:A|M. f" == "CONST complex_set_lebesgue_integral M A (\<lambda>x. f)"
 
-lemma set_measurable_continuous_on_ivl:
-  assumes "continuous_on {a..b} (f :: real \<Rightarrow> real)"
-  shows "set_borel_measurable borel {a..b} f"
-  unfolding set_borel_measurable_def
-  by (rule borel_measurable_continuous_on_indicator[OF _ assms]) simp
+lemma set_measurable_continuous_on:
+  fixes f g :: "'a::topological_space \<Rightarrow> 'b::real_normed_vector"
+  shows "A \<in> sets borel \<Longrightarrow> continuous_on A f \<Longrightarrow> set_borel_measurable borel A f"
+  by (meson borel_measurable_continuous_on_indicator
+      set_borel_measurable_def)
 
 section \<open>NN Set Integrals\<close>