doc-src/IsarRef/Thy/Generic.thy
changeset 42617 77d239840285
parent 42596 6c621a9d612a
child 42626 6ac8c55c657e
--- a/doc-src/IsarRef/Thy/Generic.thy	Mon May 02 16:33:21 2011 +0200
+++ b/doc-src/IsarRef/Thy/Generic.thy	Mon May 02 17:06:40 2011 +0200
@@ -284,7 +284,7 @@
   @{rail "
     (@@{method rule_tac} | @@{method erule_tac} | @@{method drule_tac} |
       @@{method frule_tac} | @@{method cut_tac} | @@{method thin_tac}) @{syntax goalspec}?
-    ( insts @{syntax thmref} | @{syntax thmrefs} )
+    ( dynamic_insts @'in' @{syntax thmref} | @{syntax thmrefs} )
     ;
     @@{method subgoal_tac} @{syntax goalspec}? (@{syntax prop} +)
     ;
@@ -295,8 +295,8 @@
     (@@{method tactic} | @@{method raw_tactic}) @{syntax text}
     ;
 
-    insts: ((@{syntax name} '=' @{syntax term}) + @'and') @'in'
-  "} % FIXME check use of insts
+    dynamic_insts: ((@{syntax name} '=' @{syntax term}) + @'and')
+  "}
 
 \begin{description}