src/HOL/BNF_Least_Fixpoint.thy
changeset 58182 82478e6c60cb
parent 58179 2de7b0313de3
child 58211 c1f3fa32d322
--- a/src/HOL/BNF_Least_Fixpoint.thy	Thu Sep 04 09:02:43 2014 +0200
+++ b/src/HOL/BNF_Least_Fixpoint.thy	Thu Sep 04 11:20:59 2014 +0200
@@ -188,6 +188,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"
 
 lemma size_bool[code]: "size (b\<Colon>bool) = 0"
   by (cases b) auto