author | bulwahn |
Thu, 02 Jun 2011 08:55:08 +0200 | |
changeset 43146 | 09f74fda1b1d |
parent 43124 | fdb7e1d5f762 |
child 43241 | 93b1183e43e5 |
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 |
43146 | 16 |
Dlist_Cset |
24281 | 17 |
Eval_Witness |
28952
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
haftmann
parents:
28668
diff
changeset
|
18 |
Float |
29688 | 19 |
Formal_Power_Series |
31761
3585bebe49a8
Added Library/Fraction_Field.thy: The fraction field of any integral
chaieb
parents:
31379
diff
changeset
|
20 |
Fraction_Field |
29986 | 21 |
FrechetDeriv |
40672
abd4e7358847
replaced misleading Fset/fset name -- these do not stand for finite sets
haftmann
parents:
40349
diff
changeset
|
22 |
Cset |
21256 | 23 |
FuncSet |
38622 | 24 |
Function_Algebras |
29879 | 25 |
Fundamental_Theorem_Algebra |
37665 | 26 |
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
|
27 |
Infinite_Set |
29993 | 28 |
Inner_Product |
35032
7efe662e41b4
separate library theory for type classes combining lattices with various algebraic structures
haftmann
parents:
34020
diff
changeset
|
29 |
Lattice_Algebras |
30326
a01b2de0e3e1
constructive version of Cantor's first diagonalization argument
haftmann
parents:
30261
diff
changeset
|
30 |
Lattice_Syntax |
26173 | 31 |
ListVector |
31990 | 32 |
Kleene_Algebra |
29708 | 33 |
Mapping |
37790 | 34 |
Monad_Syntax |
37023 | 35 |
More_List |
15131 | 36 |
Multiset |
37 |
Nat_Infinity |
|
38 |
Nested_Environment |
|
24332
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents:
24281
diff
changeset
|
39 |
Numeral_Type |
15470 | 40 |
OptionalSugar |
26232 | 41 |
Option_ord |
15131 | 42 |
Permutation |
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 |
30019
a2f19e0a28b2
add theory of products as real vector spaces to Library
huffman
parents:
30018
diff
changeset
|
46 |
Product_Vector |
35222
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
47 |
Quotient_List |
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
48 |
Quotient_Option |
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
49 |
Quotient_Product |
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
50 |
Quotient_Sum |
4f1fba00f66d
Initial version of HOL quotient package.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
35100
diff
changeset
|
51 |
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
|
52 |
Quotient_Type |
21635
32f3e1127de2
added Ramsey.thy to Library imports, to include it in the daily builds
krauss
parents:
21256
diff
changeset
|
53 |
Ramsey |
29650 | 54 |
Reflection |
43124 | 55 |
RBT_Mapping |
38622 | 56 |
Set_Algebras |
33084 | 57 |
SML_Quickcheck |
21256 | 58 |
State_Monad |
41474 | 59 |
Sum_of_Squares |
33649
854173fcd21c
added a tabled implementation of the reflexive transitive closure
bulwahn
parents:
33356
diff
changeset
|
60 |
Transitive_Closure_Table |
29504 | 61 |
Univ_Poly |
15131 | 62 |
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
|
63 |
Zorn |
15131 | 64 |
begin |
10253 | 65 |
end |
66 |
(*>*) |