src/HOL/Analysis/Homeomorphism.thy
changeset 77200 8f2e6186408f
parent 72569 d56e4eeae967
child 78248 740b23f1138a
--- a/src/HOL/Analysis/Homeomorphism.thy	Sun Feb 05 20:09:39 2023 +0100
+++ b/src/HOL/Analysis/Homeomorphism.thy	Mon Feb 06 15:41:23 2023 +0000
@@ -1017,6 +1017,14 @@
                         pairwise disjnt v \<and>
                         (\<forall>u \<in> v. \<exists>q. homeomorphism u T p q)))"
 
+lemma covering_spaceI [intro?]:
+  assumes "continuous_on c p" "p ` c = S"
+          "\<And>x. x \<in> S \<Longrightarrow> \<exists>T. x \<in> T \<and> openin (top_of_set S) T \<and>
+                             (\<exists>v. \<Union>v = c \<inter> p -` T \<and> (\<forall>u \<in> v. openin (top_of_set c) u) \<and>
+                             pairwise disjnt v \<and> (\<forall>u \<in> v. \<exists>q. homeomorphism u T p q))"
+  shows "covering_space c p S"
+  using assms unfolding covering_space_def by auto
+
 lemma covering_space_imp_continuous: "covering_space c p S \<Longrightarrow> continuous_on c p"
   by (simp add: covering_space_def)