src/HOL/Probability/Probability_Mass_Function.thy
changeset 69529 4ab9657b3257
parent 69313 b021008c5397
child 69597 ff784d5a5bfb
--- a/src/HOL/Probability/Probability_Mass_Function.thy	Fri Dec 28 19:01:35 2018 +0100
+++ b/src/HOL/Probability/Probability_Mass_Function.thy	Sat Dec 29 15:43:53 2018 +0100
@@ -848,7 +848,7 @@
         by (simp add: sums_unique)
     next
       show "uniform_limit A (\<lambda>n a. \<Sum>i<n. ?f i a) (\<lambda>a. (\<Sum> n. ?f n a)) sequentially"
-      proof (rule weierstrass_m_test)
+      proof (rule Weierstrass_m_test)
         fix n a assume "a\<in>A"
         then show "norm (?f n a) \<le> pmf (map_pmf (to_nat_on M) M) n * B"
           using bnd by (auto intro!: mult_mono simp: from_nat_into set_pmf_not_empty)