src/HOL/Quickcheck_Exhaustive.thy
changeset 51126 df86080de4cb
parent 49948 744934b818c7
child 51143 0a2371e7ced3
equal deleted inserted replaced
51125:f90874d3a246 51126:df86080de4cb
     1 (* Author: Lukas Bulwahn, TU Muenchen *)
     1 (* Author: Lukas Bulwahn, TU Muenchen *)
     2 
     2 
     3 header {* A simple counterexample generator performing exhaustive testing *}
     3 header {* A simple counterexample generator performing exhaustive testing *}
     4 
     4 
     5 theory Quickcheck_Exhaustive
     5 theory Quickcheck_Exhaustive
     6 imports Quickcheck
     6 imports Quickcheck_Random
     7 keywords "quickcheck_generator" :: thy_decl
     7 keywords "quickcheck_generator" :: thy_decl
     8 begin
     8 begin
     9 
     9 
    10 subsection {* basic operations for exhaustive generators *}
    10 subsection {* basic operations for exhaustive generators *}
    11 
    11