src/HOL/Hilbert_Choice.thy
changeset 44921 58eef4843641
parent 44890 22f665a2e91c
child 45607 16b4f5774621
--- a/src/HOL/Hilbert_Choice.thy	Tue Sep 13 08:21:51 2011 -0700
+++ b/src/HOL/Hilbert_Choice.thy	Tue Sep 13 17:07:33 2011 -0700
@@ -123,7 +123,7 @@
 by (simp add:inv_into_f_eq)
 
 lemma inj_imp_inv_eq: "[| inj f; ALL x. f(g x) = x |] ==> inv f = g"
-by (blast intro: ext inv_into_f_eq)
+  by (blast intro: inv_into_f_eq)
 
 text{*But is it useful?*}
 lemma inj_transfer:
@@ -286,7 +286,7 @@
   hence "?f'' a = a'"
     using `a \<in> A` 1 3 by (auto simp add: f_inv_into_f bij_betw_def)
   moreover have "f a = a'" using assms 2 3
-    by (auto simp add: inv_into_f_f bij_betw_def)
+    by (auto simp add: bij_betw_def)
   ultimately show "?f'' a = f a" by simp
 qed