src/Tools/Auto_Counterexample.thy
author blanchet
Wed, 28 Oct 2009 17:43:43 +0100
changeset 33561 ab01b72715ef
permissions -rw-r--r--
introduced Auto Nitpick in addition to Auto Quickcheck; this required generalizing the theorem hook used by Quickcheck, following a suggestion by Florian

(*  Title:   Tools/Auto_Counterexample.thy
    Author:  Jasmin Blanchette, TU Muenchen

Counterexample Search Unit (do not abbreviate!).
*)

header {* Counterexample Search Unit *}

theory Auto_Counterexample
imports Pure
uses
  "~~/src/Tools/auto_counterexample.ML"
begin

end