src/HOL/Library/Library.thy
author haftmann
Fri, 12 Oct 2007 08:21:09 +0200
changeset 24994 c385c4eabb3b
parent 24626 85eceef2edc7
child 25315 6ff4305d2f7c
permissions -rw-r--r--
consolidated naming conventions for code generator theories
wenzelm@20809
     1
(* $Id$ *)
wenzelm@10253
     2
(*<*)
nipkow@15131
     3
theory Library
nipkow@15140
     4
imports
haftmann@24197
     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@24994
    11
  Code_Index
haftmann@24994
    12
  Code_Message
wenzelm@21256
    13
  Coinductive_List
wenzelm@21256
    14
  Commutative_Ring
nipkow@15131
    15
  Continuity
haftmann@23854
    16
  Efficient_Nat
haftmann@24626
    17
  (*Eval*)
haftmann@24281
    18
  Eval_Witness
haftmann@23854
    19
  Executable_Set
wenzelm@21256
    20
  FuncSet
wenzelm@21256
    21
  GCD
wenzelm@21256
    22
  Infinite_Set
nipkow@15131
    23
  Multiset
nipkow@15131
    24
  NatPair
nipkow@15131
    25
  Nat_Infinity
nipkow@15131
    26
  Nested_Environment
kleing@24332
    27
  Numeral_Type
nipkow@15470
    28
  OptionalSugar
wenzelm@21256
    29
  Parity
nipkow@15131
    30
  Permutation
haftmann@24994
    31
  Code_Integer
haftmann@24994
    32
  Code_Char_chr
nipkow@15131
    33
  Primes
nipkow@24615
    34
  Quicksort
nipkow@15131
    35
  Quotient
krauss@21635
    36
  Ramsey
wenzelm@21256
    37
  State_Monad
krauss@22359
    38
  Size_Change_Termination
nipkow@15131
    39
  While_Combinator
nipkow@15131
    40
  Word
nipkow@15131
    41
  Zorn
nipkow@15131
    42
begin
wenzelm@10253
    43
end
wenzelm@10253
    44
(*>*)