author | haftmann |
Mon, 21 Aug 2006 11:02:39 +0200 | |
changeset 20400 | 0ad2f3bbd4f0 |
parent 19605 | 67e6b4759b37 |
child 20809 | 6c4fd0b4b63a |
permissions | -rw-r--r-- |
10253 | 1 |
(*<*) |
15131 | 2 |
theory Library |
15140 | 3 |
imports |
16908
d374530bfaaa
Added two new theories to HOL/Library: SetsAndFunctions.thy and BigO.thy
avigad
parents:
16109
diff
changeset
|
4 |
BigO |
15131 | 5 |
Continuity |
15324 | 6 |
EfficientNat |
17633 | 7 |
ExecutableSet |
19605 | 8 |
ExecutableRat |
20400 | 9 |
MLString |
15131 | 10 |
FuncSet |
11 |
Multiset |
|
12 |
NatPair |
|
13 |
Nat_Infinity |
|
14 |
Nested_Environment |
|
15470 | 15 |
OptionalSugar |
15131 | 16 |
Permutation |
17 |
Primes |
|
18 |
Quotient |
|
19 |
While_Combinator |
|
20 |
Word |
|
21 |
Zorn |
|
15731 | 22 |
Char_ord |
17516 | 23 |
Commutative_Ring |
18397 | 24 |
Coinductive_List |
19234 | 25 |
AssocList |
15131 | 26 |
begin |
10253 | 27 |
end |
28 |
(*>*) |