src/HOL/Nitpick_Examples/Mini_Nits.thy
changeset 48891 c0eafbd55de3
parent 45970 b6d0cff57d96
child 51272 9c8d63b4b6be
--- a/src/HOL/Nitpick_Examples/Mini_Nits.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Nitpick_Examples/Mini_Nits.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -9,9 +9,10 @@
 
 theory Mini_Nits
 imports Main
-uses "minipick.ML"
 begin
 
+ML_file "minipick.ML"
+
 nitpick_params [verbose, sat_solver = MiniSat_JNI, max_threads = 1]
 
 nitpick_params [total_consts = smart]