doc-src/TutorialI/Trie/Trie.thy
changeset 16417 9bc16273c2d4
parent 15905 0a4cc9b113c7
child 17555 23c4a349feff
--- 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