| author | sultana | 
| Wed, 19 Feb 2014 15:57:02 +0000 | |
| changeset 55586 | c94f1a72d9c5 | 
| parent 55159 | 608c157d743d | 
| child 56020 | f92479477c52 | 
| permissions | -rw-r--r-- | 
| 10253 | 1 | (*<*) | 
| 15131 | 2 | theory Library | 
| 15140 | 3 | imports | 
| 51161 
6ed12ae3b3e1
attempt to re-establish conventions which theories are loaded into the grand unified library theory;
 haftmann parents: 
50134diff
changeset | 4 | AList | 
| 16908 
d374530bfaaa
Added two new theories to HOL/Library: SetsAndFunctions.thy and BigO.thy
 avigad parents: 
16109diff
changeset | 5 | BigO | 
| 29994 
6ca6b6bd6e15
add formalization of a type of integers mod 2 to Library
 huffman parents: 
29993diff
changeset | 6 | Bit | 
| 55075 | 7 | BNF_Decl | 
| 24332 
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
 kleing parents: 
24281diff
changeset | 8 | Boolean_Algebra | 
| 21256 | 9 | Char_ord | 
| 15131 | 10 | Continuity | 
| 29026 | 11 | ContNotDenum | 
| 36648 | 12 | Convex | 
| 26170 | 13 | Countable | 
| 55075 | 14 | Countable_Set_Type | 
| 48427 
571cb1df0768
library theories for debugging and parallel computing using code generation towards Isabelle/ML
 haftmann parents: 
48283diff
changeset | 15 | Debug | 
| 50087 | 16 | Diagonal_Subsequence | 
| 48283 | 17 | Dlist | 
| 51542 | 18 | Extended | 
| 19 | Extended_Nat | |
| 20 | Extended_Real | |
| 48028 | 21 | FinFun | 
| 28952 
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
 haftmann parents: 
28668diff
changeset | 22 | Float | 
| 29688 | 23 | Formal_Power_Series | 
| 31761 
3585bebe49a8
Added Library/Fraction_Field.thy: The fraction field of any integral
 chaieb parents: 
31379diff
changeset | 24 | Fraction_Field | 
| 53953 | 25 | FSet | 
| 21256 | 26 | FuncSet | 
| 48188 | 27 | Function_Division | 
| 51263 
31e786e0e6a7
turned example into library for comparing growth of functions
 haftmann parents: 
51174diff
changeset | 28 | Function_Growth | 
| 29879 | 29 | Fundamental_Theorem_Algebra | 
| 37665 | 30 | Indicator_Function | 
| 27475 
61b979a2c820
add Infinite_Set and Zorn back in (since they are no longer included in main HOL image)
 huffman parents: 
27368diff
changeset | 31 | Infinite_Set | 
| 29993 | 32 | Inner_Product | 
| 51161 
6ed12ae3b3e1
attempt to re-establish conventions which theories are loaded into the grand unified library theory;
 haftmann parents: 
50134diff
changeset | 33 | IArray | 
| 35032 
7efe662e41b4
separate library theory for type classes combining lattices with various algebraic structures
 haftmann parents: 
34020diff
changeset | 34 | Lattice_Algebras | 
| 30326 
a01b2de0e3e1
constructive version of Cantor's first diagonalization argument
 haftmann parents: 
30261diff
changeset | 35 | Lattice_Syntax | 
| 26173 | 36 | ListVector | 
| 31990 | 37 | Kleene_Algebra | 
| 29708 | 38 | Mapping | 
| 37790 | 39 | Monad_Syntax | 
| 15131 | 40 | Multiset | 
| 24332 
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
 kleing parents: 
24281diff
changeset | 41 | Numeral_Type | 
| 15470 | 42 | OptionalSugar | 
| 26232 | 43 | Option_ord | 
| 48427 
571cb1df0768
library theories for debugging and parallel computing using code generation towards Isabelle/ML
 haftmann parents: 
48283diff
changeset | 44 | Parallel | 
| 15131 | 45 | Permutation | 
| 44227 
78e033e8ba05
get Library/Permutations.thy compiled and working again
 huffman parents: 
44014diff
changeset | 46 | Permutations | 
| 29985 
57975b45ab70
split polynomial-related stuff from Deriv.thy into Library/Poly_Deriv.thy
 huffman parents: 
29879diff
changeset | 47 | Poly_Deriv | 
| 29987 | 48 | Polynomial | 
| 31060 
75d7c7cc8bdb
added theory for explicit equivalence relation in preorders
 haftmann parents: 
30326diff
changeset | 49 | Preorder | 
| 30019 
a2f19e0a28b2
add theory of products as real vector spaces to Library
 huffman parents: 
30018diff
changeset | 50 | Product_Vector | 
| 35222 
4f1fba00f66d
Initial version of HOL quotient package.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
35100diff
changeset | 51 | Quotient_List | 
| 
4f1fba00f66d
Initial version of HOL quotient package.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
35100diff
changeset | 52 | Quotient_Option | 
| 
4f1fba00f66d
Initial version of HOL quotient package.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
35100diff
changeset | 53 | Quotient_Product | 
| 45074 | 54 | Quotient_Set | 
| 35222 
4f1fba00f66d
Initial version of HOL quotient package.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
35100diff
changeset | 55 | Quotient_Sum | 
| 
4f1fba00f66d
Initial version of HOL quotient package.
 Cezary Kaliszyk <kaliszyk@in.tum.de> parents: 
35100diff
changeset | 56 | 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: 
35091diff
changeset | 57 | Quotient_Type | 
| 21635 
32f3e1127de2
added Ramsey.thy to Library imports, to include it in the daily builds
 krauss parents: 
21256diff
changeset | 58 | Ramsey | 
| 29650 | 59 | Reflection | 
| 44818 
27ba81ad0890
theory of saturated naturals contributed by Peter Gammie
 haftmann parents: 
44561diff
changeset | 60 | Saturated | 
| 38622 | 61 | Set_Algebras | 
| 21256 | 62 | State_Monad | 
| 51161 
6ed12ae3b3e1
attempt to re-establish conventions which theories are loaded into the grand unified library theory;
 haftmann parents: 
50134diff
changeset | 63 | Sublist | 
| 41474 | 64 | Sum_of_Squares | 
| 33649 
854173fcd21c
added a tabled implementation of the reflexive transitive closure
 bulwahn parents: 
33356diff
changeset | 65 | Transitive_Closure_Table | 
| 15131 | 66 | While_Combinator | 
| 67 | begin | |
| 10253 | 68 | end | 
| 69 | (*>*) |