| 35953 |      1 | (* Author: Lukas Bulwahn, TU Muenchen *)
 | 
|  |      2 | 
 | 
|  |      3 | header {* A Prototype of Quickcheck based on the Predicate Compiler *}
 | 
|  |      4 | 
 | 
|  |      5 | theory Predicate_Compile_Quickcheck
 | 
|  |      6 | imports Main Predicate_Compile_Alternative_Defs
 | 
|  |      7 | uses "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML"
 | 
|  |      8 | begin
 | 
|  |      9 | 
 | 
| 36026 |     10 | setup {* Quickcheck.add_generator ("predicate_compile_wo_ff", Predicate_Compile_Quickcheck.quickcheck_compile_term
 | 
|  |     11 |   Predicate_Compile_Aux.New_Pos_Random_DSeq false true 4) *}
 | 
|  |     12 | setup {* Quickcheck.add_generator ("predicate_compile_ff_fs",
 | 
|  |     13 |   Predicate_Compile_Quickcheck.quickcheck_compile_term Predicate_Compile_Aux.New_Pos_Random_DSeq true true 4) *}
 | 
|  |     14 | setup {* Quickcheck.add_generator ("predicate_compile_ff_nofs",
 | 
|  |     15 |   Predicate_Compile_Quickcheck.quickcheck_compile_term Predicate_Compile_Aux.New_Pos_Random_DSeq true false 4) *}
 | 
| 35953 |     16 | 
 | 
|  |     17 | end |