src/HOL/Analysis/Bochner_Integration.thy
changeset 70136 f03a01a18c6e
parent 69739 8b47c021666e
child 70271 f7630118814c
--- a/src/HOL/Analysis/Bochner_Integration.thy	Fri Apr 12 19:48:29 2019 +0200
+++ b/src/HOL/Analysis/Bochner_Integration.thy	Fri Apr 12 22:09:25 2019 +0200
@@ -309,7 +309,7 @@
   then show "emeasure M {y \<in> space M. f y \<noteq> 0} \<noteq> \<infinity>" by simp
 qed fact
 
-definition%important simple_bochner_integral :: "'a measure \<Rightarrow> ('a \<Rightarrow> 'b::real_vector) \<Rightarrow> 'b" where
+definition\<^marker>\<open>tag important\<close> simple_bochner_integral :: "'a measure \<Rightarrow> ('a \<Rightarrow> 'b::real_vector) \<Rightarrow> 'b" where
   "simple_bochner_integral M f = (\<Sum>y\<in>f`space M. measure M {x\<in>space M. f x = y} *\<^sub>R y)"
 
 proposition simple_bochner_integral_partition:
@@ -895,7 +895,7 @@
 
 end
 
-definition%important lebesgue_integral ("integral\<^sup>L") where
+definition\<^marker>\<open>tag important\<close> lebesgue_integral ("integral\<^sup>L") where
   "integral\<^sup>L M f = (if \<exists>x. has_bochner_integral M f x then THE x. has_bochner_integral M f x else 0)"
 
 syntax