src/HOL/ex/Codegenerator_Candidates.thy
author bulwahn
Tue, 03 Nov 2009 10:36:20 +0100
changeset 33405 5c1928d5db38
parent 33356 9157d0f9f00e
child 33500 22e5725be1f3
permissions -rw-r--r--
adding testcases for code inlining, sets and numerals to the example files of the predicate compiler and its quickcheck prototype; disabling length example


(* Author: Florian Haftmann, TU Muenchen *)

header {* A huge collection of equations to generate code from *}

theory Codegenerator_Candidates
imports
  Complex_Main
  AssocList
  Binomial
  Fset
  Enum
  List_Prefix
  Nat_Infinity
  Nested_Environment
  Option_ord
  Permutation
  "~~/src/HOL/Number_Theory/Primes"
  Product_ord
  SetsAndFunctions
  Tree
  While_Combinator
  Word
  "~~/src/HOL/Decision_Procs/Commutative_Ring_Complete"
  "~~/src/HOL/ex/Records"
begin

(*avoid popular infix*)
code_reserved SML upto

end