src/HOL/Probability/Probability_Space.thy
changeset 41097 a1abfa4e2b44
parent 41095 c335d880ff82
child 41544 c3b977fee8a3
equal deleted inserted replaced
41096:843c40bbc379 41097:a1abfa4e2b44
  1067   qed
  1067   qed
  1068   from choice[OF this] guess g .. note g = this
  1068   from choice[OF this] guess g .. note g = this
  1069 
  1069 
  1070   show "\<exists>g\<in>borel_measurable M'. \<forall>x\<in>space M. Z x = g (Y x)"
  1070   show "\<exists>g\<in>borel_measurable M'. \<forall>x\<in>space M. Z x = g (Y x)"
  1071   proof (intro ballI bexI)
  1071   proof (intro ballI bexI)
  1072     show "(SUP i. g i) \<in> borel_measurable M'"
  1072     show "(\<lambda>x. SUP i. g i x) \<in> borel_measurable M'"
  1073       using g by (auto intro: M'.borel_measurable_simple_function)
  1073       using g by (auto intro: M'.borel_measurable_simple_function)
  1074     fix x assume "x \<in> space M"
  1074     fix x assume "x \<in> space M"
  1075     have "Z x = (SUP i. f i) x" using `f \<up> Z` unfolding isoton_def by simp
  1075     have "Z x = (SUP i. f i) x" using `f \<up> Z` unfolding isoton_def by simp
  1076     also have "\<dots> = (SUP i. g i) (Y x)" unfolding SUPR_fun_expand
  1076     also have "\<dots> = (SUP i. g i (Y x))" unfolding SUPR_apply
  1077       using g `x \<in> space M` by simp
  1077       using g `x \<in> space M` by simp
  1078     finally show "Z x = (SUP i. g i) (Y x)" .
  1078     finally show "Z x = (SUP i. g i (Y x))" .
  1079   qed
  1079   qed
  1080 qed
  1080 qed
  1081 
  1081 
  1082 end
  1082 end