src/HOL/Probability/Borel_Space.thy
changeset 50001 382bd3173584
parent 49774 dfa8ddb874ce
child 50002 ce0d316b5b44
equal deleted inserted replaced
50000:cfe8ee8a1371 50001:382bd3173584
    88 lemma borel_measurable_indicator[simp, intro!]:
    88 lemma borel_measurable_indicator[simp, intro!]:
    89   assumes A: "A \<in> sets M"
    89   assumes A: "A \<in> sets M"
    90   shows "indicator A \<in> borel_measurable M"
    90   shows "indicator A \<in> borel_measurable M"
    91   unfolding indicator_def [abs_def] using A
    91   unfolding indicator_def [abs_def] using A
    92   by (auto intro!: measurable_If_set)
    92   by (auto intro!: measurable_If_set)
       
    93 
       
    94 lemma borel_measurable_indicator': 
       
    95   "{x\<in>space M. x \<in> A} \<in> sets M \<Longrightarrow> indicator A \<in> borel_measurable M"
       
    96   unfolding indicator_def[abs_def]
       
    97   by (auto intro!: measurable_If)
    93 
    98 
    94 lemma borel_measurable_indicator_iff:
    99 lemma borel_measurable_indicator_iff:
    95   "(indicator A :: 'a \<Rightarrow> 'x::{t1_space, zero_neq_one}) \<in> borel_measurable M \<longleftrightarrow> A \<inter> space M \<in> sets M"
   100   "(indicator A :: 'a \<Rightarrow> 'x::{t1_space, zero_neq_one}) \<in> borel_measurable M \<longleftrightarrow> A \<inter> space M \<in> sets M"
    96     (is "?I \<in> borel_measurable M \<longleftrightarrow> _")
   101     (is "?I \<in> borel_measurable M \<longleftrightarrow> _")
    97 proof
   102 proof