src/HOL/Probability/Levy.thy
changeset 66447 a1f5c5c26fa6
parent 65064 a4abec71279a
child 67682 00c436488398
equal deleted inserted replaced
66445:407de0768126 66447:a1f5c5c26fa6
   498   have tight: "tight M"
   498   have tight: "tight M"
   499     by (auto simp: tight_def intro: assms tight_aux)
   499     by (auto simp: tight_def intro: assms tight_aux)
   500   show ?thesis
   500   show ?thesis
   501   proof (rule tight_subseq_weak_converge [OF real_distr_M real_distr_M' tight])
   501   proof (rule tight_subseq_weak_converge [OF real_distr_M real_distr_M' tight])
   502     fix s \<nu>
   502     fix s \<nu>
   503     assume s: "subseq s"
   503     assume s: "strict_mono (s :: nat \<Rightarrow> nat)"
   504     assume nu: "weak_conv_m (M \<circ> s) \<nu>"
   504     assume nu: "weak_conv_m (M \<circ> s) \<nu>"
   505     assume *: "real_distribution \<nu>"
   505     assume *: "real_distribution \<nu>"
   506     have 2: "\<And>n. real_distribution ((M \<circ> s) n)" unfolding comp_def by (rule assms)
   506     have 2: "\<And>n. real_distribution ((M \<circ> s) n)" unfolding comp_def by (rule assms)
   507     have 3: "\<And>t. (\<lambda>n. char ((M \<circ> s) n) t) \<longlonglongrightarrow> char \<nu> t" by (intro levy_continuity1 [OF 2 * nu])
   507     have 3: "\<And>t. (\<lambda>n. char ((M \<circ> s) n) t) \<longlonglongrightarrow> char \<nu> t" by (intro levy_continuity1 [OF 2 * nu])
   508     have 4: "\<And>t. (\<lambda>n. char ((M \<circ> s) n) t) = ((\<lambda>n. char (M n) t) \<circ> s)" by (rule ext, simp)
   508     have 4: "\<And>t. (\<lambda>n. char ((M \<circ> s) n) t) = ((\<lambda>n. char (M n) t) \<circ> s)" by (rule ext, simp)