diff -r 6061ae1f90f2 -r 9bc16273c2d4 doc-src/TutorialI/Trie/Trie.thy --- a/doc-src/TutorialI/Trie/Trie.thy Fri Jun 17 11:35:35 2005 +0200 +++ b/doc-src/TutorialI/Trie/Trie.thy Fri Jun 17 16:12:49 2005 +0200 @@ -1,5 +1,5 @@ (*<*) -theory Trie = Main:; +theory Trie imports Main begin; (*>*) text{* To minimize running time, each node of a trie should contain an array that maps