src/HOL/Library/Reflection.thy
changeset 48891 c0eafbd55de3
parent 46765 07f9eda810b3
child 51542 738598beeb26
--- a/src/HOL/Library/Reflection.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Library/Reflection.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -6,11 +6,11 @@
 
 theory Reflection
 imports Main
-uses
-  "~~/src/HOL/Library/reify_data.ML"
-  "~~/src/HOL/Library/reflection.ML"
 begin
 
+ML_file "~~/src/HOL/Library/reify_data.ML"
+ML_file "~~/src/HOL/Library/reflection.ML"
+
 setup {* Reify_Data.setup *}
 
 method_setup reify = {*