src/HOL/Probability/Projective_Limit.thy
changeset 69712 dc85b5b3a532
parent 69260 0a9688695a1b
child 74362 0135a0c77b64
equal deleted inserted replaced
69711:82a604715919 69712:dc85b5b3a532
   258       by (subst mu_G_spec) (auto intro!: sets.Diff)
   258       by (subst mu_G_spec) (auto intro!: sets.Diff)
   259     ultimately
   259     ultimately
   260     have "\<mu>G (Z n) - \<mu>G (Y n) = \<mu>G (Z n - Y n)"
   260     have "\<mu>G (Z n) - \<mu>G (Y n) = \<mu>G (Z n - Y n)"
   261       using J J_mono K_sets \<open>n \<ge> 1\<close>
   261       using J J_mono K_sets \<open>n \<ge> 1\<close>
   262       by (simp only: emeasure_eq_measure Z_def)
   262       by (simp only: emeasure_eq_measure Z_def)
   263          (auto dest!: bspec[where x=n] intro!: measure_Diff[symmetric] set_mp[OF K_B]
   263          (auto dest!: bspec[where x=n] intro!: measure_Diff[symmetric] subsetD[OF K_B]
   264                intro!: arg_cong[where f=ennreal]
   264                intro!: arg_cong[where f=ennreal]
   265                simp: extensional_restrict emeasure_eq_measure prod_emb_iff sets_P space_P
   265                simp: extensional_restrict emeasure_eq_measure prod_emb_iff sets_P space_P
   266                      ennreal_minus measure_nonneg)
   266                      ennreal_minus measure_nonneg)
   267     also have subs: "Z n - Y n \<subseteq> (\<Union>i\<in>{1..n}. (Z i - Z' i))"
   267     also have subs: "Z n - Y n \<subseteq> (\<Union>i\<in>{1..n}. (Z i - Z' i))"
   268       using \<open>n \<ge> 1\<close> unfolding Y_def UN_extend_simps(7) by (intro UN_mono Diff_mono Z_mono order_refl) auto
   268       using \<open>n \<ge> 1\<close> unfolding Y_def UN_extend_simps(7) by (intro UN_mono Diff_mono Z_mono order_refl) auto