src/HOL/Library/Library.thy
author haftmann
Fri, 18 Jul 2008 18:25:56 +0200
changeset 27652 818666de6c24
parent 27475 61b979a2c820
child 28098 c92850d2d16c
permissions -rw-r--r--
refined code generator setup for rational numbers; more simplification rules for rational numbers
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@26170
    22
  Eval
haftmann@24281
    23
  Eval_Witness
haftmann@23854
    24
  Executable_Set
haftmann@27298
    25
  "../Real/Float"
wenzelm@21256
    26
  FuncSet
haftmann@26170
    27
  Imperative_HOL
huffman@27475
    28
  Infinite_Set
wenzelm@26173
    29
  ListVector
nipkow@15131
    30
  Multiset
nipkow@15131
    31
  NatPair
nipkow@15131
    32
  Nat_Infinity
nipkow@15131
    33
  Nested_Environment
kleing@24332
    34
  Numeral_Type
nipkow@15470
    35
  OptionalSugar
haftmann@26232
    36
  Option_ord
nipkow@15131
    37
  Permutation
nipkow@15131
    38
  Primes
nipkow@24615
    39
  Quicksort
nipkow@15131
    40
  Quotient
krauss@21635
    41
  Ramsey
krauss@26192
    42
  RBT
wenzelm@21256
    43
  State_Monad
nipkow@15131
    44
  While_Combinator
nipkow@15131
    45
  Word
huffman@27475
    46
  Zorn
nipkow@15131
    47
begin
wenzelm@10253
    48
end
wenzelm@10253
    49
(*>*)