author | haftmann |
Thu, 07 May 2009 12:17:17 +0200 | |
changeset 31060 | 75d7c7cc8bdb |
parent 30326 | a01b2de0e3e1 |
child 31117 | 527ba4a37843 |
permissions | -rw-r--r-- |
10253 | 1 |
(*<*) |
15131 | 2 |
theory Library |
15140 | 3 |
imports |
27652
818666de6c24
refined code generator setup for rational numbers; more simplification rules for rational numbers
haftmann
parents:
27475
diff
changeset
|
4 |
Abstract_Rat |
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 |
29994
6ca6b6bd6e15
add formalization of a type of integers mod 2 to Library
huffman
parents:
29993
diff
changeset
|
8 |
Bit |
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
24281
diff
changeset
|
9 |
Boolean_Algebra |
21256 | 10 |
Char_ord |
26170 | 11 |
Code_Char_chr |
24994
c385c4eabb3b
consolidated naming conventions for code generator theories
haftmann
parents:
24626
diff
changeset
|
12 |
Code_Index |
26170 | 13 |
Code_Integer |
21256 | 14 |
Coinductive_List |
15 |
Commutative_Ring |
|
15131 | 16 |
Continuity |
29026 | 17 |
ContNotDenum |
26170 | 18 |
Countable |
29847 | 19 |
Determinants |
30326
a01b2de0e3e1
constructive version of Cantor's first diagonalization argument
haftmann
parents:
30261
diff
changeset
|
20 |
Diagonalize |
23854 | 21 |
Efficient_Nat |
26348 | 22 |
Enum |
24281 | 23 |
Eval_Witness |
23854 | 24 |
Executable_Set |
28952
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
28668
diff
changeset
|
25 |
Float |
29688 | 26 |
Formal_Power_Series |
29986 | 27 |
FrechetDeriv |
21256 | 28 |
FuncSet |
29879 | 29 |
Fundamental_Theorem_Algebra |
27475
61b979a2c820
add Infinite_Set and Zorn back in (since they are no longer included in main HOL image)
huffman
parents:
27368
diff
changeset
|
30 |
Infinite_Set |
29993 | 31 |
Inner_Product |
30326
a01b2de0e3e1
constructive version of Cantor's first diagonalization argument
haftmann
parents:
30261
diff
changeset
|
32 |
Lattice_Syntax |
26173 | 33 |
ListVector |
29708 | 34 |
Mapping |
15131 | 35 |
Multiset |
36 |
Nat_Infinity |
|
37 |
Nested_Environment |
|
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
24281
diff
changeset
|
38 |
Numeral_Type |
15470 | 39 |
OptionalSugar |
26232 | 40 |
Option_ord |
15131 | 41 |
Permutation |
28668
e79e196039a1
fixed and reactivated HOL/Library/Pocklington.thy -- by Mark Hillebrand;
wenzelm
parents:
28228
diff
changeset
|
42 |
Pocklington |
29985
57975b45ab70
split polynomial-related stuff from Deriv.thy into Library/Poly_Deriv.thy
huffman
parents:
29879
diff
changeset
|
43 |
Poly_Deriv |
29987 | 44 |
Polynomial |
31060
75d7c7cc8bdb
added theory for explicit equivalence relation in preorders
haftmann
parents:
30326
diff
changeset
|
45 |
Preorder |
15131 | 46 |
Primes |
30019
a2f19e0a28b2
add theory of products as real vector spaces to Library
huffman
parents:
30018
diff
changeset
|
47 |
Product_Vector |
29806 | 48 |
Quickcheck |
24615 | 49 |
Quicksort |
15131 | 50 |
Quotient |
21635
32f3e1127de2
added Ramsey.thy to Library imports, to include it in the daily builds
krauss
parents:
21256
diff
changeset
|
51 |
Ramsey |
29806 | 52 |
Random |
29650 | 53 |
Reflection |
26192
52617dca8386
new theory of red-black trees, an efficient implementation of finite maps.
krauss
parents:
26173
diff
changeset
|
54 |
RBT |
21256 | 55 |
State_Monad |
30261
4db36ab8d1c4
Added Libray dependency on Topology_Euclidean_Space
chaieb
parents:
30242
diff
changeset
|
56 |
Topology_Euclidean_Space |
29504 | 57 |
Univ_Poly |
15131 | 58 |
While_Combinator |
59 |
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
|
60 |
Zorn |
15131 | 61 |
begin |
10253 | 62 |
end |
63 |
(*>*) |