src/Doc/Isar_Ref/Generic.thy
changeset 59763 56d2c357e6b5
parent 59582 0fbed69ff081
child 59780 23b67731f4f0
--- a/src/Doc/Isar_Ref/Generic.thy	Fri Mar 20 11:53:22 2015 +0100
+++ b/src/Doc/Isar_Ref/Generic.thy	Fri Mar 20 14:48:04 2015 +0100
@@ -319,7 +319,7 @@
 
   \item @{method rule_tac} etc. do resolution of rules with explicit
   instantiation.  This works the same way as the ML tactics @{ML
-  res_inst_tac} etc.\ (see @{cite "isabelle-implementation"}).
+  Rule_Insts.res_inst_tac} etc.\ (see @{cite "isabelle-implementation"}).
 
   Multiple rules may be only given if there is no instantiation; then
   @{method rule_tac} is the same as @{ML resolve_tac} in ML (see