src/HOL/Analysis/Borel_Space.thy
changeset 69566 c41954ee87cf
parent 69517 dc20f278e8f3
child 69597 ff784d5a5bfb
--- a/src/HOL/Analysis/Borel_Space.thy	Tue Jan 01 20:57:54 2019 +0100
+++ b/src/HOL/Analysis/Borel_Space.thy	Tue Jan 01 21:47:27 2019 +0100
@@ -2140,7 +2140,7 @@
   shows "(\<lambda>x. \<bar>f x\<bar> powr p) \<in> borel_measurable M"
 unfolding powr_def by auto
 
-text \<open>The next one is a variation around \verb+measurable_restrict_space+.\<close>
+text \<open>The next one is a variation around \<open>measurable_restrict_space\<close>.\<close>
 
 lemma%unimportant measurable_restrict_space3:
   assumes "f \<in> measurable M N" and
@@ -2152,7 +2152,7 @@
       measurable_restrict_space2[of f, of "restrict_space M A", of B, of N] assms(2) space_restrict_space)
 qed
 
-text \<open>The next one is a variation around \verb+measurable_piecewise_restrict+.\<close>
+text \<open>The next one is a variation around \<open>measurable_piecewise_restrict\<close>.\<close>
 
 lemma%important measurable_piecewise_restrict2:
   assumes [measurable]: "\<And>n. A n \<in> sets M"