src/CCL/CCL.thy
changeset 59780 23b67731f4f0
parent 59763 56d2c357e6b5
child 60754 02924903a6fd
--- a/src/CCL/CCL.thy	Mon Mar 23 10:16:20 2015 +0100
+++ b/src/CCL/CCL.thy	Mon Mar 23 13:30:59 2015 +0100
@@ -476,7 +476,7 @@
 method_setup eq_coinduct3 = {*
   Scan.lift Args.name_inner_syntax >> (fn s => fn ctxt =>
     SIMPLE_METHOD'
-      (Rule_Insts.res_inst_tac ctxt [((("R", 0), Position.none), s)] @{thm eq_coinduct3}))
+      (Rule_Insts.res_inst_tac ctxt [((("R", 0), Position.none), s)] [] @{thm eq_coinduct3}))
 *}