src/LCF/LCF.thy
changeset 27239 f2f42f9fa09d
parent 27208 5fe899199f85
child 35128 c1ad622e90e4
--- a/src/LCF/LCF.thy	Mon Jun 16 17:56:08 2008 +0200
+++ b/src/LCF/LCF.thy	Mon Jun 16 22:13:39 2008 +0200
@@ -317,7 +317,7 @@
 
 ML {*
   fun induct_tac ctxt v i =
-    RuleInsts.res_inst_tac ctxt [(("f", 0), v)] @{thm induct} i THEN
+    res_inst_tac ctxt [(("f", 0), v)] @{thm induct} i THEN
     REPEAT (resolve_tac @{thms adm_lemmas} i)
 *}
 
@@ -376,7 +376,7 @@
 
 ML {*
 fun induct2_tac ctxt (f, g) i =
-  RuleInsts.res_inst_tac ctxt [(("f", 0), f), (("g", 0), g)] @{thm induct2} i THEN
+  res_inst_tac ctxt [(("f", 0), f), (("g", 0), g)] @{thm induct2} i THEN
   REPEAT(resolve_tac @{thms adm_lemmas} i)
 *}