diff -r f90874d3a246 -r df86080de4cb src/HOL/Quickcheck_Exhaustive.thy --- a/src/HOL/Quickcheck_Exhaustive.thy Thu Feb 14 17:58:28 2013 +0100 +++ b/src/HOL/Quickcheck_Exhaustive.thy Thu Feb 14 15:27:10 2013 +0100 @@ -3,7 +3,7 @@ header {* A simple counterexample generator performing exhaustive testing *} theory Quickcheck_Exhaustive -imports Quickcheck +imports Quickcheck_Random keywords "quickcheck_generator" :: thy_decl begin