src/HOL/Probability/Complete_Measure.thy
changeset 43920 cedb5cb948fd
parent 42866 b0746bd57a41
child 46731 5302e932d1e5
--- a/src/HOL/Probability/Complete_Measure.thy	Tue Jul 19 14:35:44 2011 +0200
+++ b/src/HOL/Probability/Complete_Measure.thy	Tue Jul 19 14:36:12 2011 +0200
@@ -253,7 +253,7 @@
 qed
 
 lemma (in completeable_measure_space) completion_ex_borel_measurable_pos:
-  fixes g :: "'a \<Rightarrow> extreal"
+  fixes g :: "'a \<Rightarrow> ereal"
   assumes g: "g \<in> borel_measurable completion" and "\<And>x. 0 \<le> g x"
   shows "\<exists>g'\<in>borel_measurable M. (AE x. g x = g' x)"
 proof -
@@ -279,7 +279,7 @@
 qed
 
 lemma (in completeable_measure_space) completion_ex_borel_measurable:
-  fixes g :: "'a \<Rightarrow> extreal"
+  fixes g :: "'a \<Rightarrow> ereal"
   assumes g: "g \<in> borel_measurable completion"
   shows "\<exists>g'\<in>borel_measurable M. (AE x. g x = g' x)"
 proof -