src/HOL/Quickcheck_Exhaustive.thy
changeset 41918 d2ab869f8b0b
parent 41916 80060d5f864a
child 41920 d4fb7a418152
--- a/src/HOL/Quickcheck_Exhaustive.thy	Fri Mar 11 15:21:13 2011 +0100
+++ b/src/HOL/Quickcheck_Exhaustive.thy	Fri Mar 11 15:21:13 2011 +0100
@@ -2,7 +2,7 @@
 
 header {* A simple counterexample generator performing exhaustive testing *}
 
-theory Quickcheck_Exhautive
+theory Quickcheck_Exhaustive
 imports Quickcheck
 uses ("Tools/exhaustive_generators.ML")
 begin
@@ -368,9 +368,9 @@
 code_const catch_match 
   (SML "(_) handle Match => _")
 
-use "Tools/smallvalue_generators.ML"
+use "Tools/exhaustive_generators.ML"
 
-setup {* Smallvalue_Generators.setup *}
+setup {* Exhaustive_Generators.setup *}
 
 declare [[quickcheck_tester = exhaustive]]