src/HOL/Probability/Fin_Map.thy
changeset 78103 0252d635bfb2
parent 74362 0135a0c77b64
child 80768 c7723cc15de8
--- a/src/HOL/Probability/Fin_Map.thy	Tue May 16 14:16:20 2023 +0200
+++ b/src/HOL/Probability/Fin_Map.thy	Tue May 16 22:23:05 2023 +0200
@@ -232,7 +232,7 @@
       case (UN B)
       then obtain b where "x \<in> b" "b \<in> B" by auto
       hence "\<exists>a\<in>?A. a \<subseteq> b" using UN by simp
-      thus ?case using \<open>b \<in> B\<close> by blast
+      thus ?case using \<open>b \<in> B\<close> by (metis Sup_upper2)
     next
       case (Basis s)
       then obtain a b where xs: "x\<in> Pi' a b" "s = Pi' a b" "\<And>i. i\<in>a \<Longrightarrow> open (b i)" by auto