src/HOL/Codatatype/Codatatype.thy
author traytel
Tue, 04 Sep 2012 12:10:19 +0200
changeset 49109 0e5b859e1c91
parent 49075 ed769978dc8d
child 49112 4de4635d8f93
permissions -rw-r--r--
no more aliases for Local_Theory.note; use Thm.close_derivation in internal theorems;

(*  Title:      HOL/Codatatype/Codatatype.thy
    Author:     Dmitriy Traytel, TU Muenchen
    Author:     Andrei Popescu, TU Muenchen
    Author:     Jasmin Blanchette, TU Muenchen
    Copyright   2012

The (co)datatype package.
*)

header {* The (Co)datatype Package *}

theory Codatatype
imports BNF_Wrap BNF_LFP BNF_GFP
begin

end