src/HOL/HOLCF/Domain.thy
changeset 48891 c0eafbd55de3
parent 46950 d0181abdbdac
child 57945 cacb00a569e0
--- a/src/HOL/HOLCF/Domain.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/HOLCF/Domain.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -9,11 +9,6 @@
 keywords
   "domaindef" :: thy_decl and "lazy" "unsafe" and
   "domain_isomorphism" "domain" :: thy_decl
-uses
-  ("Tools/domaindef.ML")
-  ("Tools/Domain/domain_isomorphism.ML")
-  ("Tools/Domain/domain_axioms.ML")
-  ("Tools/Domain/domain.ML")
 begin
 
 default_sort "domain"
@@ -155,7 +150,7 @@
   , (@{const_name liftprj}, SOME @{typ "udom u \<rightarrow> 'a::predomain u"}) ]
 *}
 
-use "Tools/domaindef.ML"
+ML_file "Tools/domaindef.ML"
 
 subsection {* Isomorphic deflations *}
 
@@ -321,9 +316,9 @@
 
 subsection {* Setting up the domain package *}
 
-use "Tools/Domain/domain_isomorphism.ML"
-use "Tools/Domain/domain_axioms.ML"
-use "Tools/Domain/domain.ML"
+ML_file "Tools/Domain/domain_isomorphism.ML"
+ML_file "Tools/Domain/domain_axioms.ML"
+ML_file "Tools/Domain/domain.ML"
 
 setup Domain_Isomorphism.setup