src/HOL/Nitpick.thy
changeset 49989 34d0ac1bdac6
parent 48891 c0eafbd55de3
child 52641 c56b6fa636e8
--- a/src/HOL/Nitpick.thy	Wed Oct 31 11:23:21 2012 +0100
+++ b/src/HOL/Nitpick.thy	Wed Oct 31 11:23:21 2012 +0100
@@ -8,7 +8,7 @@
 header {* Nitpick: Yet Another Counterexample Generator for Isabelle/HOL *}
 
 theory Nitpick
-imports Map Quotient SAT Record
+imports Hilbert_Choice List Map Quotient Record Sledgehammer
 keywords "nitpick" :: diag and "nitpick_params" :: thy_decl
 begin