src/HOL/Codatatype/BNF_Def.thy
changeset 49282 c057e1b39f16
parent 48975 7f79f94a432c
child 49283 97809ae5f7bb
equal deleted inserted replaced
49281:3d87f4fd0d50 49282:c057e1b39f16
     6 *)
     6 *)
     7 
     7 
     8 header {* Definition of Bounded Natural Functors *}
     8 header {* Definition of Bounded Natural Functors *}
     9 
     9 
    10 theory BNF_Def
    10 theory BNF_Def
    11 imports BNF_Library
    11 imports BNF_Util
    12 keywords
    12 keywords
    13   "print_bnfs" :: diag
    13   "print_bnfs" :: diag
    14 and
    14 and
    15   "bnf_def" :: thy_goal
    15   "bnf_def" :: thy_goal
    16 uses
    16 uses