diff -r e0f68a507683 -r b021008c5397 src/HOL/Analysis/Improper_Integral.thy --- a/src/HOL/Analysis/Improper_Integral.thy Sun Nov 18 09:51:41 2018 +0100 +++ b/src/HOL/Analysis/Improper_Integral.thy Sun Nov 18 18:07:51 2018 +0000 @@ -793,7 +793,7 @@ proof (rule sum_content_area_over_thin_division) show "snd ` S division_of \(snd ` S)" by (auto intro: S tagged_partial_division_of_Union_self division_of_tagged_division) - show "UNION S snd \ cbox a b" + show "\(snd ` S) \ cbox a b" using S by force show "a \ i \ c \ i" "c \ i \ b \ i" using mem_box(2) that by blast+ @@ -987,7 +987,7 @@ proof - obtain u v where uv: "L = cbox u v" using T'_tagged \(x, L) \ A\ \A \ T''\ \T'' \ T'\ by blast - have "A tagged_division_of UNION A snd" + have "A tagged_division_of \(snd ` A)" using A_tagged tagged_partial_division_of_Union_self by auto then have "interior (K \ {x. x \ i \ c}) = {}" apply (rule tagged_division_split_left_inj [OF _ \(x,K) \ A\ \(x,L) \ A\]) @@ -1016,7 +1016,7 @@ proof - obtain u v where uv: "L = cbox u v" using T'_tagged \(x, L) \ B\ \B \ T''\ \T'' \ T'\ by blast - have "B tagged_division_of UNION B snd" + have "B tagged_division_of \(snd ` B)" using B_tagged tagged_partial_division_of_Union_self by auto then have "interior (K \ {x. c \ x \ i}) = {}" apply (rule tagged_division_split_right_inj [OF _ \(x,K) \ B\ \(x,L) \ B\])