diff -r f40bc75b2a3f -r 0252d635bfb2 src/HOL/Probability/Fin_Map.thy --- 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 \ b" "b \ B" by auto hence "\a\?A. a \ b" using UN by simp - thus ?case using \b \ B\ by blast + thus ?case using \b \ B\ by (metis Sup_upper2) next case (Basis s) then obtain a b where xs: "x\ Pi' a b" "s = Pi' a b" "\i. i\a \ open (b i)" by auto