src/HOL/Analysis/Caratheodory.thy
changeset 67682 00c436488398
parent 66804 3f9bb52082c4
child 68833 fde093888c16
--- a/src/HOL/Analysis/Caratheodory.thy	Tue Feb 20 22:04:04 2018 +0100
+++ b/src/HOL/Analysis/Caratheodory.thy	Tue Feb 20 22:25:23 2018 +0100
@@ -854,7 +854,7 @@
     { fix i assume "i \<in> I" then show "\<mu>' (G i) = \<mu> i"
       using \<mu>' by (auto intro!: inj sel) }
     show "G ` I \<subseteq> Pow \<Omega>"
-      by fact
+      by (rule space_closed)
     then show "positive (sets M) \<mu>'" "countably_additive (sets M) \<mu>'"
       using \<mu>' by (simp_all add: M sets_extend_measure measure_space_def)
   qed fact