src/LCF/LCF.thy
changeset 59780 23b67731f4f0
parent 59763 56d2c357e6b5
child 60770 240563fbf41d
--- a/src/LCF/LCF.thy	Mon Mar 23 10:16:20 2015 +0100
+++ b/src/LCF/LCF.thy	Mon Mar 23 13:30:59 2015 +0100
@@ -321,7 +321,7 @@
 method_setup induct = {*
   Scan.lift Args.name_inner_syntax >> (fn v => fn ctxt =>
     SIMPLE_METHOD' (fn i =>
-      Rule_Insts.res_inst_tac ctxt [((("f", 0), Position.none), v)] @{thm induct} i THEN
+      Rule_Insts.res_inst_tac ctxt [((("f", 0), Position.none), v)] [] @{thm induct} i THEN
       REPEAT (resolve_tac ctxt @{thms adm_lemmas} i)))
 *}
 
@@ -381,7 +381,7 @@
 ML {*
 fun induct2_tac ctxt (f, g) i =
   Rule_Insts.res_inst_tac ctxt
-    [((("f", 0), Position.none), f), ((("g", 0), Position.none), g)] @{thm induct2} i THEN
+    [((("f", 0), Position.none), f), ((("g", 0), Position.none), g)] [] @{thm induct2} i THEN
   REPEAT(resolve_tac ctxt @{thms adm_lemmas} i)
 *}