doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 45768 97be233b32ed
parent 45767 fe2fd2f76f48
parent 45766 46046d8e9659
child 45839 43a5b86bc102
equal deleted inserted replaced
45767:fe2fd2f76f48 45768:97be233b32ed
  1590       @{text quickcheck_exhaustive_active}, @{text quickcheck_random_active},
  1590       @{text quickcheck_exhaustive_active}, @{text quickcheck_random_active},
  1591       @{text quickcheck_narrowing_active} are set to true.
  1591       @{text quickcheck_narrowing_active} are set to true.
  1592     \item[@{text size}] specifies the maximum size of the search space
  1592     \item[@{text size}] specifies the maximum size of the search space
  1593     for assignment values.
  1593     for assignment values.
  1594 
  1594 
       
  1595     \item[@{text genuine_only}] sets quickcheck only to return genuine
       
  1596       counterexample, but not potentially spurious counterexamples due
       
  1597       to underspecified functions.
       
  1598     
  1595     \item[@{text eval}] takes a term or a list of terms and evaluates
  1599     \item[@{text eval}] takes a term or a list of terms and evaluates
  1596       these terms under the variable assignment found by quickcheck.
  1600       these terms under the variable assignment found by quickcheck.
  1597 
  1601 
  1598     \item[@{text iterations}] sets how many sets of assignments are
  1602     \item[@{text iterations}] sets how many sets of assignments are
  1599     generated for each particular size.
  1603     generated for each particular size.
  1607     instantiate type variables.
  1611     instantiate type variables.
  1608 
  1612 
  1609     \item[@{text report}] if set quickcheck reports how many tests
  1613     \item[@{text report}] if set quickcheck reports how many tests
  1610     fulfilled the preconditions.
  1614     fulfilled the preconditions.
  1611 
  1615 
  1612     \item[@{text quiet}] if not set quickcheck informs about the
  1616     \item[@{text quiet}] if set quickcheck does not output anything
  1613     current size for assignment values.
  1617     while testing.
       
  1618     
       
  1619     \item[@{text verbose}] if set quickcheck informs about the
       
  1620     current size and cardinality while testing.
  1614 
  1621 
  1615     \item[@{text expect}] can be used to check if the user's
  1622     \item[@{text expect}] can be used to check if the user's
  1616     expectation was met (@{text no_expectation}, @{text
  1623     expectation was met (@{text no_expectation}, @{text
  1617     no_counterexample}, or @{text counterexample}).
  1624     no_counterexample}, or @{text counterexample}).
  1618 
  1625