src/HOL/Analysis/Equivalence_Lebesgue_Henstock_Integration.thy
changeset 67986 b65c4a6a015e
parent 67984 adc1a992c470
child 67989 706f86afff43
equal deleted inserted replaced
67985:7811748de271 67986:b65c4a6a015e
  1333 proof -
  1333 proof -
  1334   have "measure lebesgue (S - T) = 0"
  1334   have "measure lebesgue (S - T) = 0"
  1335     using neg negligible_Un_eq negligible_imp_measure0 by blast
  1335     using neg negligible_Un_eq negligible_imp_measure0 by blast
  1336   then show ?thesis
  1336   then show ?thesis
  1337     by (metis S Un_commute add.right_neutral lmeasurable_negligible_symdiff measure_Un2 neg negligible_Un_eq negligible_imp_measure0)
  1337     by (metis S Un_commute add.right_neutral lmeasurable_negligible_symdiff measure_Un2 neg negligible_Un_eq negligible_imp_measure0)
       
  1338 qed
       
  1339 
       
  1340 text\<open>Negligibility of image under non-injective linear map\<close>
       
  1341 lemma negligible_Union_nat:
       
  1342   assumes "\<And>n::nat. negligible(S n)"
       
  1343   shows "negligible(\<Union>n. S n)"
       
  1344 proof -
       
  1345   have "negligible (\<Union>m\<le>k. S m)" for k
       
  1346     using assms by blast
       
  1347   then have 0:  "integral UNIV (indicat_real (\<Union>m\<le>k. S m)) = 0"
       
  1348     and 1: "(indicat_real (\<Union>m\<le>k. S m)) integrable_on UNIV" for k
       
  1349     by (auto simp: negligible has_integral_iff)
       
  1350   have 2: "\<And>k x. indicat_real (\<Union>m\<le>k. S m) x \<le> (indicat_real (\<Union>m\<le>Suc k. S m) x)"
       
  1351     by (simp add: indicator_def)
       
  1352   have 3: "\<And>x. (\<lambda>k. indicat_real (\<Union>m\<le>k. S m) x) \<longlonglongrightarrow> (indicat_real (\<Union>n. S n) x)"
       
  1353     by (force simp: indicator_def eventually_sequentially intro: Lim_eventually)
       
  1354   have 4: "bounded (range (\<lambda>k. integral UNIV (indicat_real (\<Union>m\<le>k. S m))))"
       
  1355     by (simp add: 0 image_def)
       
  1356   have *: "indicat_real (\<Union>n. S n) integrable_on UNIV \<and>
       
  1357         (\<lambda>k. integral UNIV (indicat_real (\<Union>m\<le>k. S m))) \<longlonglongrightarrow> (integral UNIV (indicat_real (\<Union>n. S n)))"
       
  1358     by (intro monotone_convergence_increasing 1 2 3 4)
       
  1359   then have "integral UNIV (indicat_real (\<Union>n. S n)) = (0::real)"
       
  1360     using LIMSEQ_unique by (auto simp: 0)
       
  1361   then show ?thesis
       
  1362     using * by (simp add: negligible_UNIV has_integral_iff)
  1338 qed
  1363 qed
  1339 
  1364 
  1340 subsection \<open>Negligibility of a Lipschitz image of a negligible set\<close>
  1365 subsection \<open>Negligibility of a Lipschitz image of a negligible set\<close>
  1341 
  1366 
  1342 text\<open>The bound will be eliminated by a sort of onion argument\<close>
  1367 text\<open>The bound will be eliminated by a sort of onion argument\<close>