src/HOL/PreList.thy
changeset 10733 59f82484e000
parent 10680 26e4aecf3207
child 11787 85b3735a51e1
--- a/src/HOL/PreList.thy	Sat Dec 23 22:50:19 2000 +0100
+++ b/src/HOL/PreList.thy	Sat Dec 23 22:50:39 2000 +0100
@@ -1,6 +1,6 @@
 (*  Title:      HOL/PreList.thy
     ID:         $Id$
-    Author:     Tobias Nipkow
+    Author:     Tobias Nipkow and Markus Wenzel
     Copyright   2000 TU Muenchen
 
 A basis for building theory List on. Is defined separately to serve as a
@@ -19,6 +19,7 @@
 
 (*belongs to theory Datatype_Universe; hides popular names *)
 hide const Node Atom Leaf Numb Lim Funs Split Case
+hide type node item
 
 
 (* generic summation indexed over nat *)