--- a/src/HOL/Library/Library.thy Wed Nov 08 22:24:54 2006 +0100
+++ b/src/HOL/Library/Library.thy Wed Nov 08 23:11:13 2006 +0100
@@ -2,30 +2,33 @@
(*<*)
theory Library
imports
+ AssocList
BigO
+ Binomial
+ Char_ord
+ Coinductive_List
+ Commutative_Ring
Continuity
EfficientNat
+ ExecutableRat
ExecutableSet
- ExecutableRat
+ FuncSet
+ GCD
+ Infinite_Set
MLString
- FuncSet
Multiset
NatPair
Nat_Infinity
Nested_Environment
OptionalSugar
+ Parity
Permutation
Primes
Quotient
+ State_Monad
While_Combinator
Word
Zorn
- Char_ord
- Commutative_Ring
- Coinductive_List
- AssocList
- Infinite_Set
- State_Monad
begin
end
(*>*)