src/HOL/ex/Interpretation_with_Defs.thy
changeset 48891 c0eafbd55de3
parent 48644 70a5d78e8326
child 55599 6535c537b243
--- a/src/HOL/ex/Interpretation_with_Defs.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/ex/Interpretation_with_Defs.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -6,7 +6,8 @@
 
 theory Interpretation_with_Defs
 imports Pure
-uses "~~/src/Tools/interpretation_with_defs.ML"
 begin
 
+ML_file "~~/src/Tools/interpretation_with_defs.ML"
+
 end