src/HOL/Hilbert_Choice.thy
changeset 26105 ae06618225ec
parent 26072 f65a7fa2da6c
child 26347 105f55201077
--- a/src/HOL/Hilbert_Choice.thy	Wed Feb 20 23:24:38 2008 +0100
+++ b/src/HOL/Hilbert_Choice.thy	Thu Feb 21 17:33:58 2008 +0100
@@ -268,6 +268,11 @@
   apply (simp add: Inv_mem)
   done
 
+lemma bij_betw_Inv: "bij_betw f A B \<Longrightarrow> bij_betw (Inv A f) B A"
+  apply (auto simp add: bij_betw_def inj_on_Inv Inv_mem)
+  apply (simp add: image_compose [symmetric] o_def)
+  apply (simp add: image_def Inv_f_f)
+  done
 
 subsection {*Other Consequences of Hilbert's Epsilon*}