src/HOL/Library/Library.thy
changeset 14706 71590b7733b7
parent 14494 48ae8d678d88
child 15131 c69542757a4d
--- a/src/HOL/Library/Library.thy	Thu May 06 12:43:00 2004 +0200
+++ b/src/HOL/Library/Library.thy	Thu May 06 14:14:18 2004 +0200
@@ -1,16 +1,18 @@
 (*<*)
 theory Library =
-  Quotient +
-  Nat_Infinity +
-  List_Prefix +
-  Nested_Environment +
   Accessible_Part +
   Continuity +
+  FuncSet +
+  List_Prefix +
   Multiset +
-  Permutation +
   NatPair +
+  Nat_Infinity +
+  Nested_Environment +
+  Permutation +
   Primes +
+  Quotient +
+  While_Combinator +
   Word +
-  While_Combinator:
+  Zorn:
 end
 (*>*)