src/HOL/Cardinals/Fun_More_Base.thy
changeset 51764 67f05cb13e08
parent 49310 6e30078de4f0
--- a/src/HOL/Cardinals/Fun_More_Base.thy	Wed Apr 24 16:21:23 2013 +0200
+++ b/src/HOL/Cardinals/Fun_More_Base.thy	Wed Apr 24 16:43:19 2013 +0200
@@ -32,7 +32,7 @@
         IM1: "f ` A \<le> A'" and IM2: "f' ` A' \<le> A"
 shows "bij_betw f A A'"
 using assms
-proof(unfold bij_betw_def inj_on_def, auto)
+proof(unfold bij_betw_def inj_on_def, safe)
   fix a b assume *: "a \<in> A" "b \<in> A" and **: "f a = f b"
   have "a = f'(f a) \<and> b = f'(f b)" using * LEFT by simp
   with ** show "a = b" by simp