src/HOL/Library/Library.thy
author haftmann
Wed, 03 Dec 2008 15:58:44 +0100
changeset 28952 15a4b2cf8c34
parent 28668 e79e196039a1
child 29026 5fbaa05f637f
permissions -rw-r--r--
made repository layout more coherent with logical distribution structure; stripped some $Id$s
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
wenzelm@21256
    14
  Coinductive_List
wenzelm@21256
    15
  Commutative_Ring
nipkow@15131
    16
  Continuity
haftmann@26170
    17
  Countable
chaieb@26157
    18
  Dense_Linear_Order
haftmann@23854
    19
  Efficient_Nat
haftmann@26348
    20
  Enum
haftmann@24281
    21
  Eval_Witness
haftmann@23854
    22
  Executable_Set
haftmann@28952
    23
  Float
wenzelm@21256
    24
  FuncSet
haftmann@26170
    25
  Imperative_HOL
huffman@27475
    26
  Infinite_Set
wenzelm@26173
    27
  ListVector
nipkow@15131
    28
  Multiset
nipkow@15131
    29
  Nat_Infinity
nipkow@15131
    30
  Nested_Environment
kleing@24332
    31
  Numeral_Type
nipkow@15470
    32
  OptionalSugar
haftmann@26232
    33
  Option_ord
nipkow@15131
    34
  Permutation
wenzelm@28668
    35
  Pocklington
nipkow@15131
    36
  Primes
nipkow@24615
    37
  Quicksort
nipkow@15131
    38
  Quotient
krauss@21635
    39
  Ramsey
krauss@26192
    40
  RBT
wenzelm@21256
    41
  State_Monad
nipkow@15131
    42
  While_Combinator
nipkow@15131
    43
  Word
huffman@27475
    44
  Zorn
nipkow@15131
    45
begin
wenzelm@10253
    46
end
wenzelm@10253
    47
(*>*)