src/HOL/Analysis/Sigma_Algebra.thy
changeset 69712 dc85b5b3a532
parent 69676 56acd449da41
child 69768 7e4966eaf781
--- a/src/HOL/Analysis/Sigma_Algebra.thy	Tue Jan 22 10:50:47 2019 +0000
+++ b/src/HOL/Analysis/Sigma_Algebra.thy	Tue Jan 22 12:00:16 2019 +0000
@@ -275,7 +275,7 @@
   hence "\<Union>X = (\<Union>n. from_nat_into X n)"
     using assms by (auto cong del: SUP_cong)
   also have "\<dots> \<in> M" using assms
-    by (auto intro!: countable_nat_UN) (metis \<open>X \<noteq> {}\<close> from_nat_into set_mp)
+    by (auto intro!: countable_nat_UN) (metis \<open>X \<noteq> {}\<close> from_nat_into subsetD)
   finally show ?thesis .
 qed simp