src/HOL/Analysis/Abstract_Topology.thy
changeset 78200 264f2b69d09c
parent 78127 24b70433c2e8
child 78248 740b23f1138a
equal deleted inserted replaced
78198:c268def0784b 78200:264f2b69d09c
  3031 subsection\<open>Relation of homeomorphism between topological spaces\<close>
  3031 subsection\<open>Relation of homeomorphism between topological spaces\<close>
  3032 
  3032 
  3033 definition homeomorphic_space (infixr "homeomorphic'_space" 50)
  3033 definition homeomorphic_space (infixr "homeomorphic'_space" 50)
  3034   where "X homeomorphic_space Y \<equiv> \<exists>f g. homeomorphic_maps X Y f g"
  3034   where "X homeomorphic_space Y \<equiv> \<exists>f g. homeomorphic_maps X Y f g"
  3035 
  3035 
  3036 lemma homeomorphic_space_refl: "X homeomorphic_space X"
  3036 lemma homeomorphic_space_refl [iff]: "X homeomorphic_space X"
  3037   by (meson homeomorphic_maps_id homeomorphic_space_def)
  3037   by (meson homeomorphic_maps_id homeomorphic_space_def)
  3038 
  3038 
  3039 lemma homeomorphic_space_sym:
  3039 lemma homeomorphic_space_sym:
  3040    "X homeomorphic_space Y \<longleftrightarrow> Y homeomorphic_space X"
  3040    "X homeomorphic_space Y \<longleftrightarrow> Y homeomorphic_space X"
  3041   unfolding homeomorphic_space_def by (metis homeomorphic_maps_sym)
  3041   unfolding homeomorphic_space_def by (metis homeomorphic_maps_sym)