src/HOL/Probability/Borel_Space.thy
changeset 61880 ff4d33058566
parent 61808 fc1556774cfe
child 61969 e01015e49041
equal deleted inserted replaced
61879:e4f9d8f094fe 61880:ff4d33058566
  1465     done
  1465     done
  1466   then show ?thesis
  1466   then show ?thesis
  1467     by simp
  1467     by simp
  1468 qed
  1468 qed
  1469 
  1469 
       
  1470 lemma is_real_interval:
       
  1471   assumes S: "is_interval S"
       
  1472   shows "\<exists>a b::real. S = {} \<or> S = UNIV \<or> S = {..<b} \<or> S = {..b} \<or> S = {a<..} \<or> S = {a..} \<or>
       
  1473     S = {a<..<b} \<or> S = {a<..b} \<or> S = {a..<b} \<or> S = {a..b}"
       
  1474   using S unfolding is_interval_1 by (blast intro: interval_cases)
       
  1475 
       
  1476 lemma real_interval_borel_measurable:
       
  1477   assumes "is_interval (S::real set)"
       
  1478   shows "S \<in> sets borel"
       
  1479 proof -
       
  1480   from assms is_real_interval have "\<exists>a b::real. S = {} \<or> S = UNIV \<or> S = {..<b} \<or> S = {..b} \<or>
       
  1481     S = {a<..} \<or> S = {a..} \<or> S = {a<..<b} \<or> S = {a<..b} \<or> S = {a..<b} \<or> S = {a..b}" by auto
       
  1482   then guess a ..
       
  1483   then guess b ..
       
  1484   thus ?thesis
       
  1485     by auto
       
  1486 qed
       
  1487 
       
  1488 lemma borel_measurable_mono:
       
  1489   fixes f :: "real \<Rightarrow> real"
       
  1490   assumes "mono f"
       
  1491   shows "f \<in> borel_measurable borel"
       
  1492 proof (subst borel_measurable_iff_ge, auto simp add:)
       
  1493   fix a :: real
       
  1494   have "is_interval {w. a \<le> f w}"
       
  1495     unfolding is_interval_1 using assms by (auto dest: monoD intro: order.trans)
       
  1496   thus "{w. a \<le> f w} \<in> sets borel" using real_interval_borel_measurable by auto  
       
  1497 qed
       
  1498 
  1470 no_notation
  1499 no_notation
  1471   eucl_less (infix "<e" 50)
  1500   eucl_less (infix "<e" 50)
  1472 
  1501 
  1473 end
  1502 end