doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 46592 d5d49bd4a7b4
parent 46498 2754784e9153
child 46628 e1bdcbe04b83
equal deleted inserted replaced
46591:1116909ef176 46592:d5d49bd4a7b4
  1641     @{command_def (HOL) "refute"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\
  1641     @{command_def (HOL) "refute"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\
  1642     @{command_def (HOL) "nitpick"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\
  1642     @{command_def (HOL) "nitpick"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\
  1643     @{command_def (HOL) "quickcheck_params"} & : & @{text "theory \<rightarrow> theory"} \\
  1643     @{command_def (HOL) "quickcheck_params"} & : & @{text "theory \<rightarrow> theory"} \\
  1644     @{command_def (HOL) "refute_params"} & : & @{text "theory \<rightarrow> theory"} \\
  1644     @{command_def (HOL) "refute_params"} & : & @{text "theory \<rightarrow> theory"} \\
  1645     @{command_def (HOL) "nitpick_params"} & : & @{text "theory \<rightarrow> theory"} \\
  1645     @{command_def (HOL) "nitpick_params"} & : & @{text "theory \<rightarrow> theory"} \\
  1646     @{command_def (HOL) "quickcheck_generator"} & : & @{text "theory \<rightarrow> theory"}
  1646     @{command_def (HOL) "quickcheck_generator"} & : & @{text "theory \<rightarrow> theory"} \\
       
  1647     @{command_def (HOL) "find_unused_assms"} & : & @{text "context \<rightarrow>"}
  1647   \end{matharray}
  1648   \end{matharray}
  1648 
  1649 
  1649   @{rail "
  1650   @{rail "
  1650     @@{command (HOL) value} ( '[' name ']' )? modes? @{syntax term}
  1651     @@{command (HOL) value} ( '[' name ']' )? modes? @{syntax term}
  1651     ;
  1652     ;
  1658     ;
  1659     ;
  1659 
  1660 
  1660     (@@{command (HOL) quickcheck_params} | @@{command (HOL) refute_params} |
  1661     (@@{command (HOL) quickcheck_params} | @@{command (HOL) refute_params} |
  1661       @@{command (HOL) nitpick_params}) ( '[' args ']' )?
  1662       @@{command (HOL) nitpick_params}) ( '[' args ']' )?
  1662     ;
  1663     ;
       
  1664 
  1663     @@{command (HOL) quickcheck_generator} typeconstructor \\
  1665     @@{command (HOL) quickcheck_generator} typeconstructor \\
  1664       'operations:' ( @{syntax term} +)
  1666       'operations:' ( @{syntax term} +)
       
  1667     ;
       
  1668 
       
  1669     @@{command (HOL) find_unused_assms} theoryname?
  1665     ;
  1670     ;
  1666 
  1671 
  1667     modes: '(' (@{syntax name} +) ')'
  1672     modes: '(' (@{syntax name} +) ')'
  1668     ;
  1673     ;
  1669 
  1674 
  1741     instantiate type variables.
  1746     instantiate type variables.
  1742 
  1747 
  1743     \item[@{text report}] if set quickcheck reports how many tests
  1748     \item[@{text report}] if set quickcheck reports how many tests
  1744     fulfilled the preconditions.
  1749     fulfilled the preconditions.
  1745 
  1750 
       
  1751     \item[@{text use_subtype}] if set quickcheck automatically lifts
       
  1752     conjectures to registered subtypes if possible, and tests the
       
  1753     lifted conjecture.
       
  1754 
  1746     \item[@{text quiet}] if set quickcheck does not output anything
  1755     \item[@{text quiet}] if set quickcheck does not output anything
  1747     while testing.
  1756     while testing.
  1748     
  1757     
  1749     \item[@{text verbose}] if set quickcheck informs about the current
  1758     \item[@{text verbose}] if set quickcheck informs about the current
  1750     size and cardinality while testing.
  1759     size and cardinality while testing.
  1803   counterexamples using a reduction to first-order relational
  1812   counterexamples using a reduction to first-order relational
  1804   logic. See the Nitpick manual \cite{isabelle-nitpick} for details.
  1813   logic. See the Nitpick manual \cite{isabelle-nitpick} for details.
  1805 
  1814 
  1806   \item @{command (HOL) "nitpick_params"} changes @{command (HOL)
  1815   \item @{command (HOL) "nitpick_params"} changes @{command (HOL)
  1807   "nitpick"} configuration options persistently.
  1816   "nitpick"} configuration options persistently.
       
  1817 
       
  1818   \item @{command (HOL) "find_unused_assms"} finds potentially superfluous
       
  1819   assumptions in theorems using quickcheck.
       
  1820   It takes the theory name to be checked for superfluous assumptions as
       
  1821   optional argument. If not provided, it checks the current theory.
       
  1822   Options to the internal quickcheck invocations can be changed with
       
  1823   common configuration declarations.
  1808 
  1824 
  1809   \end{description}
  1825   \end{description}
  1810 *}
  1826 *}
  1811 
  1827 
  1812 
  1828