src/HOL/Codatatype/BNF.thy
changeset 49509 163914705f8d
parent 49309 f20b24214ac2
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Codatatype/BNF.thy	Fri Sep 21 16:34:40 2012 +0200
@@ -0,0 +1,16 @@
+(*  Title:      HOL/BNF/BNF.thy
+    Author:     Dmitriy Traytel, TU Muenchen
+    Author:     Andrei Popescu, TU Muenchen
+    Author:     Jasmin Blanchette, TU Muenchen
+    Copyright   2012
+
+Bounded natural functors for (co)datatypes.
+*)
+
+header {* Bounded Natural Functors for (Co)datatypes *}
+
+theory BNF
+imports More_BNFs
+begin
+
+end