src/HOL/UNITY/UNITY_Main.thy
changeset 48891 c0eafbd55de3
parent 42795 66fcc9882784
child 51717 9e7d1c139569
--- a/src/HOL/UNITY/UNITY_Main.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/UNITY/UNITY_Main.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -7,9 +7,10 @@
 
 theory UNITY_Main
 imports Detects PPROD Follows ProgressSets
-uses "UNITY_tactics.ML"
 begin
 
+ML_file "UNITY_tactics.ML"
+
 method_setup safety = {*
     Scan.succeed (SIMPLE_METHOD' o constrains_tac) *}
     "for proving safety properties"