doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 45758 6210c350d88b
parent 45701 615da8b8d758
child 45766 46046d8e9659
equal deleted inserted replaced
45757:e32dd098f57a 45758:6210c350d88b
  1592       @{text quickcheck_exhaustive_active}, @{text quickcheck_random_active},
  1592       @{text quickcheck_exhaustive_active}, @{text quickcheck_random_active},
  1593       @{text quickcheck_narrowing_active} are set to true.
  1593       @{text quickcheck_narrowing_active} are set to true.
  1594     \item[@{text size}] specifies the maximum size of the search space
  1594     \item[@{text size}] specifies the maximum size of the search space
  1595     for assignment values.
  1595     for assignment values.
  1596 
  1596 
       
  1597     \item[@{text genuine_only}] sets quickcheck only to return genuine
       
  1598       counterexample, but not potentially spurious counterexamples due
       
  1599       to underspecified functions.
       
  1600     
  1597     \item[@{text eval}] takes a term or a list of terms and evaluates
  1601     \item[@{text eval}] takes a term or a list of terms and evaluates
  1598       these terms under the variable assignment found by quickcheck.
  1602       these terms under the variable assignment found by quickcheck.
  1599 
  1603 
  1600     \item[@{text iterations}] sets how many sets of assignments are
  1604     \item[@{text iterations}] sets how many sets of assignments are
  1601     generated for each particular size.
  1605     generated for each particular size.