| author | berghofe | 
| Wed, 07 Feb 2007 17:41:11 +0100 | |
| changeset 22270 | 4ccb7e6be929 | 
| parent 21635 | 32f3e1127de2 | 
| child 22359 | 94a794672c8b | 
| permissions | -rw-r--r-- | 
| 20809 | 1 | (* $Id$ *) | 
| 10253 | 2 | (*<*) | 
| 15131 | 3 | theory Library | 
| 15140 | 4 | imports | 
| 21256 | 5 | AssocList | 
| 16908 
d374530bfaaa
Added two new theories to HOL/Library: SetsAndFunctions.thy and BigO.thy
 avigad parents: 
16109diff
changeset | 6 | BigO | 
| 21256 | 7 | Binomial | 
| 8 | Char_ord | |
| 9 | Coinductive_List | |
| 10 | Commutative_Ring | |
| 15131 | 11 | Continuity | 
| 15324 | 12 | EfficientNat | 
| 21256 | 13 | ExecutableRat | 
| 17633 | 14 | ExecutableSet | 
| 21256 | 15 | FuncSet | 
| 16 | GCD | |
| 17 | Infinite_Set | |
| 20400 | 18 | MLString | 
| 15131 | 19 | Multiset | 
| 20 | NatPair | |
| 21 | Nat_Infinity | |
| 22 | Nested_Environment | |
| 15470 | 23 | OptionalSugar | 
| 21256 | 24 | Parity | 
| 15131 | 25 | Permutation | 
| 26 | Primes | |
| 27 | Quotient | |
| 21635 
32f3e1127de2
added Ramsey.thy to Library imports, to include it in the daily builds
 krauss parents: 
21256diff
changeset | 28 | Ramsey | 
| 21256 | 29 | State_Monad | 
| 15131 | 30 | While_Combinator | 
| 31 | Word | |
| 32 | Zorn | |
| 33 | begin | |
| 10253 | 34 | end | 
| 35 | (*>*) |