src/HOL/BNF/BNF_LFP_Compat.thy
changeset 53303 ae49b835ca01
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/BNF/BNF_LFP_Compat.thy	Fri Aug 30 11:27:23 2013 +0200
@@ -0,0 +1,18 @@
+(*  Title:      HOL/BNF/BNF_LFP_Compat.thy
+    Author:     Jasmin Blanchette, TU Muenchen
+    Copyright   2013
+
+Compatibility layer with the old datatype package.
+*)
+
+header {* Compatibility Layer with the Old Datatype Package *}
+
+theory BNF_LFP_Compat
+imports BNF_FP_N2M
+keywords
+  "datatype_compat" :: thy_goal
+begin
+
+ML_file "Tools/bnf_lfp_compat.ML"
+
+end