src/HOL/BNF/BNF_Decl.thy
changeset 55075 b3d0a02a756d
parent 55074 2b0b6f69b148
child 55076 1e73e090a514
equal deleted inserted replaced
55074:2b0b6f69b148 55075:b3d0a02a756d
     1 (*  Title:      HOL/BNF/BNF_Decl.thy
       
     2     Author:     Dmitriy Traytel, TU Muenchen
       
     3     Copyright   2013
       
     4 
       
     5 Axiomatic declaration of bounded natural functors.
       
     6 *)
       
     7 
       
     8 header {* Axiomatic declaration of Bounded Natural Functors *}
       
     9 
       
    10 theory BNF_Decl
       
    11 imports BNF_Def
       
    12 keywords
       
    13   "bnf_decl" :: thy_decl
       
    14 begin
       
    15 
       
    16 ML_file "Tools/bnf_decl.ML"
       
    17 
       
    18 end