src/FOL/FOL.thy
changeset 30549 d2d7874648bd
parent 28856 5e009a80fe6d
child 31974 e81979a703a4
--- a/src/FOL/FOL.thy	Mon Mar 16 17:51:24 2009 +0100
+++ b/src/FOL/FOL.thy	Mon Mar 16 18:24:30 2009 +0100
@@ -73,9 +73,10 @@
   fun case_tac ctxt a = res_inst_tac ctxt [(("P", 0), a)] @{thm case_split}
 *}
 
-method_setup case_tac =
-  {* Method.goal_args_ctxt Args.name_source case_tac *}
-  "case_tac emulation (dynamic instantiation!)"
+method_setup case_tac = {*
+  Args.goal_spec -- Scan.lift Args.name_source >>
+  (fn (quant, s) => fn ctxt => SIMPLE_METHOD'' quant (case_tac ctxt s))
+*} "case_tac emulation (dynamic instantiation!)"
 
 
 (*** Special elimination rules *)