src/FOL/FOL.thy
changeset 59780 23b67731f4f0
parent 59763 56d2c357e6b5
child 59940 087d81f5213e
--- a/src/FOL/FOL.thy	Mon Mar 23 10:16:20 2015 +0100
+++ b/src/FOL/FOL.thy	Mon Mar 23 13:30:59 2015 +0100
@@ -66,13 +66,13 @@
   done
 
 ML {*
-  fun case_tac ctxt a =
-    Rule_Insts.res_inst_tac ctxt [((("P", 0), Position.none), a)] @{thm case_split}
+  fun case_tac ctxt a fixes =
+    Rule_Insts.res_inst_tac ctxt [((("P", 0), Position.none), a)] fixes @{thm case_split}
 *}
 
 method_setup case_tac = {*
-  Args.goal_spec -- Scan.lift Args.name_inner_syntax >>
-    (fn (quant, s) => fn ctxt => SIMPLE_METHOD'' quant (case_tac ctxt s))
+  Args.goal_spec -- Scan.lift (Args.name_inner_syntax -- Parse.for_fixes) >>
+    (fn (quant, (s, fixes)) => fn ctxt => SIMPLE_METHOD'' quant (case_tac ctxt s fixes))
 *} "case_tac emulation (dynamic instantiation!)"