author | blanchet |
Fri, 27 Aug 2010 15:37:03 +0200 | |
changeset 38826 | f42f425edf24 |
parent 38622 | 86fc906dcd86 |
child 40349 | 131cf8790a1c |
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 |
15131 | 11 |
Continuity |
29026 | 12 |
ContNotDenum |
36648 | 13 |
Convex |
26170 | 14 |
Countable |
30326
a01b2de0e3e1
constructive version of Cantor's first diagonalization argument
haftmann
parents:
30261
diff
changeset
|
15 |
Diagonalize |
35303 | 16 |
Dlist |
26348 | 17 |
Enum |
24281 | 18 |
Eval_Witness |
28952
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
28668
diff
changeset
|
19 |
Float |
29688 | 20 |
Formal_Power_Series |
31761
3585bebe49a8
Added Library/Fraction_Field.thy: The fraction field of any integral
chaieb
parents:
31379
diff
changeset
|
21 |
Fraction_Field |
29986 | 22 |
FrechetDeriv |
31849 | 23 |
Fset |
21256 | 24 |
FuncSet |
38622 | 25 |
Function_Algebras |
29879 | 26 |
Fundamental_Theorem_Algebra |
37665 | 27 |
Indicator_Function |
27475
61b979a2c820
add Infinite_Set and Zorn back in (since they are no longer included in main HOL image)
huffman
parents:
27368
diff
changeset
|
28 |
Infinite_Set |
29993 | 29 |
Inner_Product |
35032
7efe662e41b4
separate library theory for type classes combining lattices with various algebraic structures
haftmann
parents:
34020
diff
changeset
|
30 |
Lattice_Algebras |
30326
a01b2de0e3e1
constructive version of Cantor's first diagonalization argument
haftmann
parents:
30261
diff
changeset
|
31 |
Lattice_Syntax |
26173 | 32 |
ListVector |
31990 | 33 |
Kleene_Algebra |
29708 | 34 |
Mapping |
37790 | 35 |
Monad_Syntax |
37023 | 36 |
More_List |
15131 | 37 |
Multiset |
38 |
Nat_Infinity |
|
39 |
Nested_Environment |
|
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
24281
diff
changeset
|
40 |
Numeral_Type |
15470 | 41 |
OptionalSugar |
26232 | 42 |
Option_ord |
15131 | 43 |
Permutation |
29985
57975b45ab70
split polynomial-related stuff from Deriv.thy into Library/Poly_Deriv.thy
huffman
parents:
29879
diff
changeset
|
44 |
Poly_Deriv |
29987 | 45 |
Polynomial |
31060
75d7c7cc8bdb
added theory for explicit equivalence relation in preorders
haftmann
parents:
30326
diff
changeset
|
46 |
Preorder |
30019
a2f19e0a28b2
add theory of products as real vector spaces to Library
huffman
parents:
30018
diff
changeset
|
47 |
Product_Vector |
24615 | 48 |
Quicksort |
35222
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
49 |
Quotient_List |
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
50 |
Quotient_Option |
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
51 |
Quotient_Product |
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
52 |
Quotient_Sum |
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
53 |
Quotient_Syntax |
35100
53754ec7360b
renamed Library/Quotient.thy to Library/Quotient_Type.thy to avoid clash with new theory Quotient in Main HOL;
wenzelm
parents:
35091
diff
changeset
|
54 |
Quotient_Type |
21635
32f3e1127de2
added Ramsey.thy to Library imports, to include it in the daily builds
krauss
parents:
21256
diff
changeset
|
55 |
Ramsey |
29650 | 56 |
Reflection |
26192
52617dca8386
new theory of red-black trees, an efficient implementation of finite maps.
krauss
parents:
26173
diff
changeset
|
57 |
RBT |
38622 | 58 |
Set_Algebras |
33084 | 59 |
SML_Quickcheck |
21256 | 60 |
State_Monad |
31117
527ba4a37843
Added files Sum_Of_Squares.thy, positivstellensatz.ML and sum_of_squares.ML to Library
chaieb
parents:
31060
diff
changeset
|
61 |
Sum_Of_Squares |
33649
854173fcd21c
added a tabled implementation of the reflexive transitive closure
bulwahn
parents:
33356
diff
changeset
|
62 |
Transitive_Closure_Table |
29504 | 63 |
Univ_Poly |
15131 | 64 |
While_Combinator |
27475
61b979a2c820
add Infinite_Set and Zorn back in (since they are no longer included in main HOL image)
huffman
parents:
27368
diff
changeset
|
65 |
Zorn |
15131 | 66 |
begin |
10253 | 67 |
end |
68 |
(*>*) |