src/HOL/Quickcheck_Examples/Quickcheck_Interfaces.thy
changeset 58813 625d04d4fd2a
parent 58148 9764b994a421
child 63167 0909deb8059b
--- a/src/HOL/Quickcheck_Examples/Quickcheck_Interfaces.thy	Wed Oct 29 11:13:24 2014 +0100
+++ b/src/HOL/Quickcheck_Examples/Quickcheck_Interfaces.thy	Wed Oct 29 11:19:27 2014 +0100
@@ -11,7 +11,7 @@
 First, this requires to setup special generators for all datatypes via the following command.
 *}
 
-setup {* Exhaustive_Generators.setup_bounded_forall_datatype_interpretation *}
+setup Exhaustive_Generators.setup_bounded_forall_datatype_interpretation
 
 text {*
 Now, the function Quickcheck.mk_batch_validator : Proof.context -> term list -> (int -> bool) list option