CookBook/Package/Ind_Interface.thy
changeset 35 d5c090b9a2b1
parent 32 5bb2d29553c2
child 42 cd612b489504
--- a/CookBook/Package/Ind_Interface.thy	Mon Oct 13 17:51:09 2008 +0200
+++ b/CookBook/Package/Ind_Interface.thy	Mon Oct 13 17:51:59 2008 +0200
@@ -355,7 +355,7 @@
 Most of the time, however, we will have to deal with tokens that are not just strings.
 The parsers for the theory syntax, as well as the parsers for the argument syntax
 of proof methods and attributes use the token type @{ML_type OuterParse.token},
-which is identical to the type @{ML_type OuterLex.token}.
+which is identical to @{ML_type OuterLex.token}.
 The parser functions for the theory syntax are contained in the structure
 @{ML_struct OuterParse} defined in the file @{ML_file "Pure/Isar/outer_parse.ML"}.
 In our parser, we will use the following functions: