diff -r 5c8cfaed32e6 -r 2b04504fcb69 src/HOL/Product_Type.thy --- a/src/HOL/Product_Type.thy Tue Jun 23 12:09:14 2009 +0200 +++ b/src/HOL/Product_Type.thy Tue Jun 23 12:09:30 2009 +0200 @@ -11,7 +11,7 @@ ("Tools/split_rule.ML") ("Tools/inductive_set.ML") ("Tools/inductive_realizer.ML") - ("Tools/datatype_package/datatype_realizer.ML") + ("Tools/Datatype/datatype_realizer.ML") begin subsection {* @{typ bool} is a datatype *} @@ -399,7 +399,7 @@ by (simp add: split_def id_def) lemma split_eta: "(\(x, y). f (x, y)) = f" - -- {* Subsumes the old @{text split_Pair} when @{term f} is the identity function. *} + -- {* Subsumes the old @{text split_Pair} when @{term f} is the identity Datatype. *} by (rule ext) auto lemma split_comp: "split (f \ g) x = f (g (fst x)) (snd x)" @@ -734,7 +734,7 @@ text {* @{term prod_fun} --- action of the product functor upon - functions. + Datatypes. *} definition prod_fun :: "('a \ 'c) \ ('b \ 'd) \ 'a \ 'b \ 'c \ 'd" where @@ -1154,7 +1154,7 @@ use "Tools/inductive_set.ML" setup Inductive_Set.setup -use "Tools/datatype_package/datatype_realizer.ML" +use "Tools/Datatype/datatype_realizer.ML" setup DatatypeRealizer.setup end