bulwahn@35953: (* Author: Lukas Bulwahn, TU Muenchen *) bulwahn@35953: bulwahn@35953: header {* A Prototype of Quickcheck based on the Predicate Compiler *} bulwahn@35953: bulwahn@35953: theory Predicate_Compile_Quickcheck bulwahn@35953: imports Main Predicate_Compile_Alternative_Defs bulwahn@35953: begin bulwahn@35953: wenzelm@48891: ML_file "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML" wenzelm@48891: bulwahn@43886: setup {* Predicate_Compile_Quickcheck.setup *} bulwahn@43886: haftmann@51143: end