src/HOL/Library/Library.thy
author wenzelm
Thu, 23 Oct 2008 00:24:31 +0200
changeset 28668 e79e196039a1
parent 28228 7ebe8dc06cbb
child 28952 15a4b2cf8c34
permissions -rw-r--r--
fixed and reactivated HOL/Library/Pocklington.thy -- by Mark Hillebrand;
wenzelm@20809
     1
(* $Id$ *)
wenzelm@10253
     2
(*<*)
nipkow@15131
     3
theory Library
nipkow@15140
     4
imports
haftmann@27652
     5
  Abstract_Rat
wenzelm@21256
     6
  AssocList
avigad@16908
     7
  BigO
wenzelm@21256
     8
  Binomial
kleing@24332
     9
  Boolean_Algebra
wenzelm@21256
    10
  Char_ord
haftmann@26170
    11
  Code_Char_chr
haftmann@24994
    12
  Code_Index
haftmann@26170
    13
  Code_Integer
haftmann@24994
    14
  Code_Message
wenzelm@21256
    15
  Coinductive_List
wenzelm@21256
    16
  Commutative_Ring
nipkow@15131
    17
  Continuity
haftmann@26170
    18
  Countable
chaieb@26157
    19
  Dense_Linear_Order
haftmann@23854
    20
  Efficient_Nat
haftmann@26348
    21
  Enum
haftmann@24281
    22
  Eval_Witness
haftmann@23854
    23
  Executable_Set
haftmann@27298
    24
  "../Real/Float"
wenzelm@21256
    25
  FuncSet
haftmann@26170
    26
  Imperative_HOL
huffman@27475
    27
  Infinite_Set
wenzelm@26173
    28
  ListVector
nipkow@15131
    29
  Multiset
nipkow@15131
    30
  Nat_Infinity
nipkow@15131
    31
  Nested_Environment
kleing@24332
    32
  Numeral_Type
nipkow@15470
    33
  OptionalSugar
haftmann@26232
    34
  Option_ord
nipkow@15131
    35
  Permutation
wenzelm@28668
    36
  Pocklington
nipkow@15131
    37
  Primes
nipkow@24615
    38
  Quicksort
nipkow@15131
    39
  Quotient
krauss@21635
    40
  Ramsey
krauss@26192
    41
  RBT
wenzelm@21256
    42
  State_Monad
nipkow@15131
    43
  While_Combinator
nipkow@15131
    44
  Word
huffman@27475
    45
  Zorn
nipkow@15131
    46
begin
wenzelm@10253
    47
end
wenzelm@10253
    48
(*>*)