src/HOL/Analysis/Bochner_Integration.thy
changeset 71840 8ed78bb0b915
parent 71633 07bec530f02e
child 73253 f6bb31879698
equal deleted inserted replaced
71839:0bbe0866b7e6 71840:8ed78bb0b915
   217     proof induct
   217     proof induct
   218       case empty from set[of "{}"] show ?case
   218       case empty from set[of "{}"] show ?case
   219         by (simp add: indicator_def[abs_def])
   219         by (simp add: indicator_def[abs_def])
   220     next
   220     next
   221       case (insert x F)
   221       case (insert x F)
   222       then show ?case
   222       from insert.prems have nonneg: "x \<ge> 0" "\<And>y. y \<in> F \<Longrightarrow> y \<ge> 0"
   223         by (auto intro!: add mult set sum_nonneg split: split_indicator split_indicator_asm
   223         by simp_all
   224                  simp del: sum_mult_indicator simp: sum_nonneg_eq_0_iff)
   224       hence *: "P (\<lambda>xa. x * indicat_real {x' \<in> space M. U' i x' = x} xa)"
       
   225         by (intro mult set) auto
       
   226       have "P (\<lambda>z. x * indicat_real {x' \<in> space M. U' i x' = x} z + 
       
   227                    (\<Sum>y\<in>F. y * indicat_real {x \<in> space M. U' i x = y} z))"
       
   228         using insert(1-3)
       
   229         by (intro add * sum_nonneg mult_nonneg_nonneg)
       
   230            (auto simp: nonneg indicator_def sum_nonneg_eq_0_iff)
       
   231       thus ?case 
       
   232         using insert.hyps by (subst sum.insert) auto
   225     qed
   233     qed
   226     with U' show "P (U' i)" by simp
   234     with U' show "P (U' i)" by simp
   227   qed
   235   qed
   228 qed
   236 qed
   229 
   237