src/HOL/Codatatype/BNF_LFP.thy
changeset 49308 6190b701e4f4
parent 49074 d8af889dcbe3
child 49309 f20b24214ac2
equal deleted inserted replaced
49307:30916e44d828 49308:6190b701e4f4
     6 *)
     6 *)
     7 
     7 
     8 header {* Least Fixed Point Operation on Bounded Natural Functors *}
     8 header {* Least Fixed Point Operation on Bounded Natural Functors *}
     9 
     9 
    10 theory BNF_LFP
    10 theory BNF_LFP
    11 imports BNF_Comp
    11 imports BNF_FP
    12 keywords
    12 keywords
    13   "data_raw" :: thy_decl
    13   "data_raw" :: thy_decl and
       
    14   "data" :: thy_decl
    14 uses
    15 uses
    15   "Tools/bnf_lfp_util.ML"
    16   "Tools/bnf_lfp_util.ML"
    16   "Tools/bnf_lfp_tactics.ML"
    17   "Tools/bnf_lfp_tactics.ML"
    17   "Tools/bnf_lfp.ML"
    18   "Tools/bnf_lfp.ML"
    18 begin
    19 begin