src/HOL/Analysis/T1_Spaces.thy
changeset 75455 91c16c5ad3e9
parent 71200 3548d54ce3ee
child 77935 7f240b0dabd9
--- a/src/HOL/Analysis/T1_Spaces.thy	Wed May 11 10:42:24 2022 +0200
+++ b/src/HOL/Analysis/T1_Spaces.thy	Tue May 17 14:10:14 2022 +0100
@@ -289,7 +289,7 @@
         by metis
       with \<open>a \<notin> T\<close> compactin_subset_topspace [OF T]
       have Topen: "\<forall>W \<in> U ` T. openin X W" and Tsub: "T \<subseteq> \<Union> (U ` T)"
-        by (auto simp: )
+        by auto
       then obtain \<F> where \<F>: "finite \<F>" "\<F> \<subseteq> U ` T" and "T \<subseteq> \<Union>\<F>"
         using T unfolding compactin_def by meson
       then obtain F where F: "finite F" "F \<subseteq> T" "\<F> = U ` F" and SUF: "T \<subseteq> \<Union>(U ` F)" and "a \<notin> F"