src/HOL/ex/Codegenerator_Candidates.thy
author haftmann
Thu, 25 Jun 2009 17:07:18 +0200
changeset 31807 039893a9a77d
parent 31739 8155c4d94354
child 31849 431d8588bcad
permissions -rw-r--r--
added List_Set and Code_Set theories
haftmann@21917
     1
haftmann@31378
     2
(* Author: Florian Haftmann, TU Muenchen *)
haftmann@21917
     3
haftmann@31378
     4
header {* A huge collection of equations to generate code from *}
haftmann@31378
     5
haftmann@31378
     6
theory Codegenerator_Candidates
haftmann@21917
     7
imports
haftmann@27421
     8
  Complex_Main
haftmann@21917
     9
  AssocList
haftmann@21917
    10
  Binomial
haftmann@31807
    11
  Code_Set
haftmann@21917
    12
  Commutative_Ring
haftmann@27421
    13
  Enum
haftmann@21917
    14
  List_Prefix
haftmann@21917
    15
  Nat_Infinity
haftmann@24433
    16
  Nested_Environment
haftmann@26515
    17
  Option_ord
haftmann@21917
    18
  Permutation
haftmann@21917
    19
  Primes
haftmann@21917
    20
  Product_ord
haftmann@21917
    21
  SetsAndFunctions
haftmann@31459
    22
  Tree
haftmann@21917
    23
  While_Combinator
haftmann@21917
    24
  Word
haftmann@27421
    25
  "~~/src/HOL/ex/Commutative_Ring_Complete"
haftmann@27421
    26
  "~~/src/HOL/ex/Records"
haftmann@21917
    27
begin
haftmann@21917
    28
haftmann@31378
    29
(*avoid popular infixes*)
haftmann@31378
    30
code_reserved SML union inter upto
haftmann@31378
    31
haftmann@21917
    32
end