src/HOL/Library/FuncSet.thy
changeset 61585 a9599d3d7610
parent 61384 9f5145281888
child 61955 e96292f32c3c
equal deleted inserted replaced
61584:f06e5a5a4b46 61585:a9599d3d7610
   224   by (auto simp: restrict_def Pi_def)
   224   by (auto simp: restrict_def Pi_def)
   225 
   225 
   226 
   226 
   227 subsection \<open>Bijections Between Sets\<close>
   227 subsection \<open>Bijections Between Sets\<close>
   228 
   228 
   229 text \<open>The definition of @{const bij_betw} is in @{text "Fun.thy"}, but most of
   229 text \<open>The definition of @{const bij_betw} is in \<open>Fun.thy\<close>, but most of
   230 the theorems belong here, or need at least @{term Hilbert_Choice}.\<close>
   230 the theorems belong here, or need at least @{term Hilbert_Choice}.\<close>
   231 
   231 
   232 lemma bij_betwI:
   232 lemma bij_betwI:
   233   assumes "f \<in> A \<rightarrow> B"
   233   assumes "f \<in> A \<rightarrow> B"
   234     and "g \<in> B \<rightarrow> A"
   234     and "g \<in> B \<rightarrow> A"