src/HOL/ex/Codegenerator_Candidates.thy
author immler@in.tum.de
Wed, 03 Jun 2009 16:56:41 +0200
changeset 31409 d8537ba165b5
parent 31378 d1cbf6393964
child 31459 ae39b7b2a68a
permissions -rw-r--r--
split preparing clauses and writing problemfile; included results of count_constants in return-type of prover; optionally pass counted constants to prover; removed unused external_prover from signature


(* Author: Florian Haftmann, TU Muenchen *)

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

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

(*temporary Haskell workaround*)
declare typerep_fun_def [code inline]
declare typerep_prod_def [code inline]
declare typerep_sum_def [code inline]
declare typerep_cpoint_ext_type_def [code inline]
declare typerep_itself_def [code inline]
declare typerep_list_def [code inline]
declare typerep_option_def [code inline]
declare typerep_point_ext_type_def [code inline]
declare typerep_point'_ext_type_def [code inline]
declare typerep_point''_ext_type_def [code inline]
declare typerep_pol_def [code inline]
declare typerep_polex_def [code inline]

(*avoid popular infixes*)
code_reserved SML union inter upto

end