diff -r db9f95ca2a8f -r 313d3b697c9a src/HOL/Multivariate_Analysis/Weierstrass.thy --- a/src/HOL/Multivariate_Analysis/Weierstrass.thy Mon Apr 04 09:45:04 2016 +0200 +++ b/src/HOL/Multivariate_Analysis/Weierstrass.thy Mon Apr 04 16:52:56 2016 +0100 @@ -248,7 +248,7 @@ and pf01: "\t. t \ s-U \ pf t ` s \ {0..1}" by metis have com_sU: "compact (s-U)" - using compact closed_inter_compact U by (simp add: Diff_eq compact_inter_closed open_closed) + using compact closed_Int_compact U by (simp add: Diff_eq compact_Int_closed open_closed) have "\t. t \ s-U \ \A. open A \ A \ s = {x\s. 0 < pf t x}" apply (rule open_Collect_positive) by (metis pf continuous) @@ -451,7 +451,7 @@ then have setsum_max_0: "A \ (\x \ A. Vf x)" by blast have com_A: "compact A" using A - by (metis compact compact_inter_closed inf.absorb_iff2) + by (metis compact compact_Int_closed inf.absorb_iff2) obtain subA where subA: "subA \ A" "finite subA" "A \ (\x \ subA. Vf x)" by (blast intro: that open_Vf compactE_image [OF com_A _ setsum_max_0]) then have [simp]: "subA \ {}"