src/HOL/Fun.thy
changeset 27125 0733f575b51e
parent 27106 ff27dc6e7d05
child 27165 e1c49eb8cee6
--- a/src/HOL/Fun.thy	Tue Jun 10 19:15:17 2008 +0200
+++ b/src/HOL/Fun.thy	Tue Jun 10 19:15:18 2008 +0200
@@ -465,9 +465,8 @@
 
 lemma surj_imp_surj_swap: "surj f ==> surj (swap a b f)"
 apply (simp add: surj_def swap_def, clarify)
-apply (rule_tac P = "y = f b" in case_split_thm, blast)
-apply (rule_tac P = "y = f a" in case_split_thm, auto)
-  --{*We don't yet have @{text case_tac}*}
+apply (case_tac "y = f b", blast)
+apply (case_tac "y = f a", auto)
 done
 
 lemma surj_swap_iff [simp]: "surj (swap a b f) = surj f"