src/LCF/LCF.thy
changeset 63120 629a4c5e953e
parent 60770 240563fbf41d
child 66453 cc19f7ca2ed6
--- a/src/LCF/LCF.thy	Mon May 23 20:45:10 2016 +0200
+++ b/src/LCF/LCF.thy	Mon May 23 21:30:30 2016 +0200
@@ -319,7 +319,7 @@
   adm_not_eq_tr adm_conj adm_disj adm_imp adm_all
 
 method_setup induct = \<open>
-  Scan.lift Args.name_inner_syntax >> (fn v => fn ctxt =>
+  Scan.lift Args.embedded_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
       REPEAT (resolve_tac ctxt @{thms adm_lemmas} i)))