author | huffman |
Thu, 03 Jul 2008 18:16:40 +0200 | |
changeset 27475 | 61b979a2c820 |
parent 27368 | 9f90ac19e32b |
child 27652 | 818666de6c24 |
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:
16109
diff
changeset
|
6 |
BigO |
21256 | 7 |
Binomial |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
24281
diff
changeset
|
8 |
Boolean_Algebra |
21256 | 9 |
Char_ord |
26170 | 10 |
Code_Char_chr |
24994
c385c4eabb3b
consolidated naming conventions for code generator theories
haftmann
parents:
24626
diff
changeset
|
11 |
Code_Index |
26170 | 12 |
Code_Integer |
24994
c385c4eabb3b
consolidated naming conventions for code generator theories
haftmann
parents:
24626
diff
changeset
|
13 |
Code_Message |
21256 | 14 |
Coinductive_List |
15 |
Commutative_Ring |
|
15131 | 16 |
Continuity |
26170 | 17 |
Countable |
26157 | 18 |
Dense_Linear_Order |
23854 | 19 |
Efficient_Nat |
26348 | 20 |
Enum |
26170 | 21 |
Eval |
24281 | 22 |
Eval_Witness |
23854 | 23 |
Executable_Set |
27298 | 24 |
"../Real/Float" |
21256 | 25 |
FuncSet |
26170 | 26 |
Imperative_HOL |
27475
61b979a2c820
add Infinite_Set and Zorn back in (since they are no longer included in main HOL image)
huffman
parents:
27368
diff
changeset
|
27 |
Infinite_Set |
26173 | 28 |
ListVector |
15131 | 29 |
Multiset |
30 |
NatPair |
|
31 |
Nat_Infinity |
|
32 |
Nested_Environment |
|
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
24281
diff
changeset
|
33 |
Numeral_Type |
15470 | 34 |
OptionalSugar |
26232 | 35 |
Option_ord |
15131 | 36 |
Permutation |
37 |
Primes |
|
24615 | 38 |
Quicksort |
15131 | 39 |
Quotient |
21635
32f3e1127de2
added Ramsey.thy to Library imports, to include it in the daily builds
krauss
parents:
21256
diff
changeset
|
40 |
Ramsey |
26192
52617dca8386
new theory of red-black trees, an efficient implementation of finite maps.
krauss
parents:
26173
diff
changeset
|
41 |
RBT |
21256 | 42 |
State_Monad |
15131 | 43 |
While_Combinator |
44 |
Word |
|
27475
61b979a2c820
add Infinite_Set and Zorn back in (since they are no longer included in main HOL image)
huffman
parents:
27368
diff
changeset
|
45 |
Zorn |
15131 | 46 |
begin |
10253 | 47 |
end |
48 |
(*>*) |