diff -r eddcc7c726f3 -r 4a9167f377b0 src/HOL/Analysis/Equivalence_Lebesgue_Henstock_Integration.thy --- a/src/HOL/Analysis/Equivalence_Lebesgue_Henstock_Integration.thy Mon Mar 18 15:35:34 2019 +0000 +++ b/src/HOL/Analysis/Equivalence_Lebesgue_Henstock_Integration.thy Tue Mar 19 16:14:51 2019 +0000 @@ -2032,7 +2032,7 @@ subsection\Negligibility is a local property\ lemma locally_negligible_alt: - "negligible S \ (\x \ S. \U. openin (subtopology euclidean S) U \ x \ U \ negligible U)" + "negligible S \ (\x \ S. \U. openin (top_of_set S) U \ x \ U \ negligible U)" (is "_ = ?rhs") proof assume "negligible S" @@ -2040,7 +2040,7 @@ using openin_subtopology_self by blast next assume ?rhs - then obtain U where ope: "\x. x \ S \ openin (subtopology euclidean S) (U x)" + then obtain U where ope: "\x. x \ S \ openin (top_of_set S) (U x)" and cov: "\x. x \ S \ x \ U x" and neg: "\x. x \ S \ negligible (U x)" by metis @@ -4493,7 +4493,7 @@ fix a assume a: "a \ U n" and fa: "f a \ T" define V where "V \ {x. x \ U n \ f x \ T} \ ball a (1 / n / 2)" - show "\V. openin (subtopology euclidean {x \ U n. f x \ T}) V \ a \ V \ negligible V" + show "\V. openin (top_of_set {x \ U n. f x \ T}) V \ a \ V \ negligible V" proof (intro exI conjI) have noxy: "norm(x - y) \ n * norm(f x - f y)" if "x \ V" "y \ V" for x y using that unfolding U_def V_def mem_Collect_eq Int_iff mem_ball dist_norm