src/LCF/LCF.thy
changeset 58975 762ee71498fa
parent 58973 2a683fb686fd
child 58977 9576b510f6a2
equal deleted inserted replaced
58974:cbc2ac19d783 58975:762ee71498fa
   317 lemmas adm_lemmas =
   317 lemmas adm_lemmas =
   318   adm_not_free adm_eq adm_less adm_not_less
   318   adm_not_free adm_eq adm_less adm_not_less
   319   adm_not_eq_tr adm_conj adm_disj adm_imp adm_all
   319   adm_not_eq_tr adm_conj adm_disj adm_imp adm_all
   320 
   320 
   321 method_setup induct = {*
   321 method_setup induct = {*
   322   Scan.lift Args.name >> (fn v => fn ctxt =>
   322   Scan.lift Args.name_inner_syntax >> (fn v => fn ctxt =>
   323     SIMPLE_METHOD' (fn i =>
   323     SIMPLE_METHOD' (fn i =>
   324       res_inst_tac ctxt [(("f", 0), v)] @{thm induct} i THEN
   324       res_inst_tac ctxt [(("f", 0), v)] @{thm induct} i THEN
   325       REPEAT (resolve_tac @{thms adm_lemmas} i)))
   325       REPEAT (resolve_tac @{thms adm_lemmas} i)))
   326 *}
   326 *}
   327 
   327