src/Tools/Code_Generator.thy
author blanchet
Mon, 07 Dec 2009 11:46:13 +0100
changeset 34018 39f21f7bad7e
parent 33889 4328de748fb2
child 34028 1e6206763036
permissions -rw-r--r--
avoid using "prop_logic.ML" and "sat_solver.ML" twice (the other occurrence being in "FunDef.thy"); this produces two copies of the same module, with separate references etc.

(*  Title:   Tools/Code_Generator.thy
    Author:  Florian Haftmann, TU Muenchen
*)

header {* Loading the code generator modules *}

theory Code_Generator
imports Pure
uses
  "~~/src/Tools/auto_solve.ML"
  "~~/src/Tools/auto_counterexample.ML"
  "~~/src/Tools/quickcheck.ML"
  "~~/src/Tools/value.ML"
  "~~/src/Tools/Code/code_preproc.ML" 
  "~~/src/Tools/Code/code_thingol.ML"
  "~~/src/Tools/Code/code_printer.ML"
  "~~/src/Tools/Code/code_target.ML"
  "~~/src/Tools/Code/code_ml.ML"
  "~~/src/Tools/Code/code_haskell.ML"
  "~~/src/Tools/nbe.ML"
begin

setup {*
  Code_Preproc.setup
  #> Code_ML.setup
  #> Code_Haskell.setup
  #> Nbe.setup
*}

end