src/Tools/Code_Generator.thy
author blanchet
Wed, 28 Oct 2009 17:43:43 +0100
changeset 33561 ab01b72715ef
parent 31775 2b04504fcb69
child 33820 082d9bc6992d
permissions -rw-r--r--
introduced Auto Nitpick in addition to Auto Quickcheck; this required generalizing the theorem hook used by Quickcheck, following a suggestion by Florian

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

header {* Loading the code generator modules *}

theory Code_Generator
imports Auto_Counterexample
uses
  "~~/src/Tools/value.ML"
  "~~/src/Tools/quickcheck.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