src/HOL/Analysis/Lebesgue_Measure.thy
changeset 69260 0a9688695a1b
parent 69064 5840724b1d71
child 69447 b7b9cbe0bd43
--- a/src/HOL/Analysis/Lebesgue_Measure.thy	Wed Nov 07 23:03:45 2018 +0100
+++ b/src/HOL/Analysis/Lebesgue_Measure.thy	Thu Nov 08 09:11:52 2018 +0100
@@ -1189,7 +1189,7 @@
       using emeasure_bounded_finite[of "?B n"] by (auto simp: emeasure_A)
     interpret A: finite_measure ?A
       by rule fact
-    have "emeasure ?A B + ?e n > (INF U:{U. B \<subseteq> U \<and> open U}. emeasure ?A U)"
+    have "emeasure ?A B + ?e n > (INF U\<in>{U. B \<subseteq> U \<and> open U}. emeasure ?A U)"
       using \<open>0<e\<close> by (auto simp: outer_regular[OF _ finite_A B, symmetric])
     then obtain U where U: "B \<subseteq> U" "open U" and muU: "?\<mu> (?B n \<inter> B) + ?e n > ?\<mu> (?B n \<inter> U)"
       unfolding INF_less_iff by (auto simp: emeasure_A)