src/HOL/Codatatype/BNF_GFP.thy
author blanchet
Wed, 12 Sep 2012 05:21:47 +0200
changeset 49309 f20b24214ac2
parent 49308 6190b701e4f4
child 49312 c874ff5658dc
permissions -rw-r--r--
split basic BNFs into really basic ones and others, and added Andreas Lochbihler's "option" BNF

(*  Title:      HOL/Codatatype/BNF_GFP.thy
    Author:     Dmitriy Traytel, TU Muenchen
    Copyright   2012

Greatest fixed point operation on bounded natural functors.
*)

header {* Greatest Fixed Point Operation on Bounded Natural Functors *}

theory BNF_GFP
imports BNF_FP
keywords
  "codata_raw" :: thy_decl and
  "codata" :: thy_decl
begin

ML_file "Tools/bnf_gfp_util.ML"
ML_file "Tools/bnf_gfp_tactics.ML"
ML_file "Tools/bnf_gfp.ML"

end