src/HOL/BNF_Least_Fixpoint.thy
changeset 58275 280ede57a6a9
parent 58274 4a84e94e58a2
child 58276 aa1b6ea6a893
--- a/src/HOL/BNF_Least_Fixpoint.thy	Tue Sep 09 20:51:36 2014 +0200
+++ b/src/HOL/BNF_Least_Fixpoint.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -235,7 +235,7 @@
 ML_file "Tools/BNF/bnf_lfp_rec_sugar_more.ML"
 ML_file "Tools/BNF/bnf_lfp_size.ML"
 ML_file "Tools/Function/old_size.ML"
-ML_file "Tools/Old_Datatype/old_datatype_realizer.ML"
+ML_file "Tools/datatype_realizer.ML"
 
 lemma size_bool[code]: "size (b\<Colon>bool) = 0"
   by (cases b) auto