CookBook/Parsing.thy
changeset 16 5045dec52d2b
parent 4 2a69b119cdee
child 38 e21b2f888fa2
--- a/CookBook/Parsing.thy	Thu Oct 02 04:48:41 2008 -0400
+++ b/CookBook/Parsing.thy	Thu Oct 02 05:18:49 2008 -0400
@@ -635,7 +635,7 @@
   \texttt{TRYALL} (try all subgoals, failure is OK),
   \texttt{FIRSTGOAL} (try subgoals until it succeeds once), 
   \texttt{(fn tacf => tacf 4)} (subgoal 4), etc
-  (see the \texttt{Tactical} structure, \cite[Chapter 4]{ref}).
+  (see the \texttt{Tactical} structure, FIXME) %%\cite[Chapter 4]{ref}).
 
   A method is stored in a theory as indicated by:
   \begin{verbatim}