src/HOL/Probability/Borel_Space.thy
changeset 60017 b785d6d06430
parent 59658 0cc388370041
child 60150 bd773c47ad0b
--- a/src/HOL/Probability/Borel_Space.thy	Thu Apr 09 20:42:38 2015 +0200
+++ b/src/HOL/Probability/Borel_Space.thy	Sat Apr 11 11:56:40 2015 +0100
@@ -1038,7 +1038,7 @@
 
 lemma borel_measurable_ln[measurable (raw)]:
   assumes f: "f \<in> borel_measurable M"
-  shows "(\<lambda>x. ln (f x)) \<in> borel_measurable M"
+  shows "(\<lambda>x. ln (f x :: real)) \<in> borel_measurable M"
   apply (rule measurable_compose[OF f])
   apply (rule borel_measurable_continuous_countable_exceptions[of "{0}"])
   apply (auto intro!: continuous_on_ln continuous_on_id)