src/HOL/Codatatype/BNF_Def.thy
changeset 49309 f20b24214ac2
parent 49286 dde4967c9233
child 49312 c874ff5658dc
--- a/src/HOL/Codatatype/BNF_Def.thy	Wed Sep 12 05:03:18 2012 +0200
+++ b/src/HOL/Codatatype/BNF_Def.thy	Wed Sep 12 05:21:47 2012 +0200
@@ -12,9 +12,9 @@
 keywords
   "print_bnfs" :: diag and
   "bnf_def" :: thy_goal
-uses
-  "Tools/bnf_def_tactics.ML"
-  "Tools/bnf_def.ML"
 begin
 
+ML_file "Tools/bnf_def_tactics.ML"
+ML_file"Tools/bnf_def.ML"
+
 end