src/HOL/Analysis/Connected.thy
changeset 69518 bf88364c9e94
parent 69508 2a4c8a2a3f8e
child 69529 4ab9657b3257
equal deleted inserted replaced
69517:dc20f278e8f3 69518:bf88364c9e94
  3517   by (simp add: homeomorphism_def)
  3517   by (simp add: homeomorphism_def)
  3518 
  3518 
  3519 lemma homeomorphism_sym: "homeomorphism S t f g = homeomorphism t S g f"
  3519 lemma homeomorphism_sym: "homeomorphism S t f g = homeomorphism t S g f"
  3520   by (force simp: homeomorphism_def)
  3520   by (force simp: homeomorphism_def)
  3521 
  3521 
  3522 definition homeomorphic :: "'a::topological_space set \<Rightarrow> 'b::topological_space set \<Rightarrow> bool"
  3522 definition%important homeomorphic :: "'a::topological_space set \<Rightarrow> 'b::topological_space set \<Rightarrow> bool"
  3523     (infixr "homeomorphic" 60)
  3523     (infixr "homeomorphic" 60)
  3524   where "s homeomorphic t \<equiv> (\<exists>f g. homeomorphism s t f g)"
  3524   where "s homeomorphic t \<equiv> (\<exists>f g. homeomorphism s t f g)"
  3525 
  3525 
  3526 lemma homeomorphic_empty [iff]:
  3526 lemma homeomorphic_empty [iff]:
  3527      "S homeomorphic {} \<longleftrightarrow> S = {}" "{} homeomorphic S \<longleftrightarrow> S = {}"
  3527      "S homeomorphic {} \<longleftrightarrow> S = {}" "{} homeomorphic S \<longleftrightarrow> S = {}"