src/Tools/quickcheck.ML
changeset 45755 b27a06dfb2ef
parent 45730 6bd0acefaedb
child 45757 e32dd098f57a
--- a/src/Tools/quickcheck.ML	Mon Dec 05 12:35:05 2011 +0100
+++ b/src/Tools/quickcheck.ML	Mon Dec 05 12:35:06 2011 +0100
@@ -63,6 +63,8 @@
   (* basic operations *)
   val message : Proof.context -> string -> unit
   val limit : Time.time -> (bool * bool) -> (unit -> 'a) -> (unit -> 'a) -> unit -> 'a
+  val pretty_counterex : Proof.context -> bool ->
+    ((bool * (string * term) list) * (term * term) list) option -> Pretty.T
   (* testing terms and proof states *)
   val mk_batch_validator : Proof.context -> term list -> (int -> bool) list option
   val mk_batch_tester : Proof.context -> term list -> (int -> term list option) list option