src/HOL/Product_Type.thy
changeset 48891 c0eafbd55de3
parent 47988 e4b69e10b990
child 49764 9979d64b8016
--- a/src/HOL/Product_Type.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Product_Type.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -8,9 +8,6 @@
 theory Product_Type
 imports Typedef Inductive Fun
 keywords "inductive_set" "coinductive_set" :: thy_decl
-uses
-  ("Tools/split_rule.ML")
-  ("Tools/inductive_set.ML")
 begin
 
 subsection {* @{typ bool} is a datatype *}
@@ -690,7 +687,7 @@
 lemma internal_split_conv: "internal_split c (a, b) = c a b"
   by (simp only: internal_split_def split_conv)
 
-use "Tools/split_rule.ML"
+ML_file "Tools/split_rule.ML"
 setup Split_Rule.setup
 
 hide_const internal_split
@@ -1122,7 +1119,7 @@
 
 subsection {* Inductively defined sets *}
 
-use "Tools/inductive_set.ML"
+ML_file "Tools/inductive_set.ML"
 setup Inductive_Set.setup