src/HOL/Library/Predicate_Compile_Quickcheck.thy
author huffman
Tue, 02 Aug 2011 08:28:34 -0700
changeset 44019 ee784502aed5
parent 43886 bf068e758783
child 45450 dc2236b19a3d
permissions -rw-r--r--
Extended_Nat.thy: renamed iSuc to eSuc, standardized theorem names
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
35953
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     1
(* Author: Lukas Bulwahn, TU Muenchen *)
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     2
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     3
header {* A Prototype of Quickcheck based on the Predicate Compiler *}
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     4
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     5
theory Predicate_Compile_Quickcheck
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     6
imports Main Predicate_Compile_Alternative_Defs
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     7
uses "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML"
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     8
begin
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
     9
43886
bf068e758783 adapting quickcheck based on the analysis of the predicate compiler
bulwahn
parents: 39252
diff changeset
    10
setup {* Predicate_Compile_Quickcheck.setup *}
bf068e758783 adapting quickcheck based on the analysis of the predicate compiler
bulwahn
parents: 39252
diff changeset
    11
bf068e758783 adapting quickcheck based on the analysis of the predicate compiler
bulwahn
parents: 39252
diff changeset
    12
(*setup {* Context.theory_map (Quickcheck.add_generator ("predicate_compile_wo_ff", Predicate_Compile_Quickcheck.quickcheck_compile_term
39252
8f176e575a49 changing the container for the quickcheck options to a generic data
bulwahn
parents: 36026
diff changeset
    13
  Predicate_Compile_Aux.New_Pos_Random_DSeq false true 4)) *}
8f176e575a49 changing the container for the quickcheck options to a generic data
bulwahn
parents: 36026
diff changeset
    14
setup {* Context.theory_map (Quickcheck.add_generator ("predicate_compile_ff_fs",
8f176e575a49 changing the container for the quickcheck options to a generic data
bulwahn
parents: 36026
diff changeset
    15
  Predicate_Compile_Quickcheck.quickcheck_compile_term Predicate_Compile_Aux.New_Pos_Random_DSeq true true 4)) *}
8f176e575a49 changing the container for the quickcheck options to a generic data
bulwahn
parents: 36026
diff changeset
    16
setup {* Context.theory_map (Quickcheck.add_generator ("predicate_compile_ff_nofs",
8f176e575a49 changing the container for the quickcheck options to a generic data
bulwahn
parents: 36026
diff changeset
    17
  Predicate_Compile_Quickcheck.quickcheck_compile_term Predicate_Compile_Aux.New_Pos_Random_DSeq true false 4)) *}
43886
bf068e758783 adapting quickcheck based on the analysis of the predicate compiler
bulwahn
parents: 39252
diff changeset
    18
*)
35953
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
    19
0460ff79bb52 moved further predicate compile files to HOL-Library
bulwahn
parents:
diff changeset
    20
end