| author | wenzelm | 
| Fri, 28 Apr 2017 13:21:03 +0200 | |
| changeset 65604 | 637aa8e93cd7 | 
| parent 62691 | 9bfcbab7cd99 | 
| child 69605 | a96320074298 | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Library/BNF_Axiomatization.thy Author: Dmitriy Traytel, TU Muenchen Copyright 2013 Axiomatic declaration of bounded natural functors. *) section \<open>Axiomatic Declaration of Bounded Natural Functors\<close> theory BNF_Axiomatization imports Main keywords "bnf_axiomatization" :: thy_decl begin ML_file "../Tools/BNF/bnf_axiomatization.ML" end