author | wenzelm |
Tue, 23 Dec 2014 20:46:42 +0100 | |
changeset 59184 | 830bb7ddb3ab |
parent 58881 | b9556a055632 |
child 59794 | 39442248a027 |
permissions | -rw-r--r-- |
(* Title: HOL/Library/BNF_Axiomatization.thy Author: Dmitriy Traytel, TU Muenchen Copyright 2013 Axiomatic declaration of bounded natural functors. *) section {* Axiomatic declaration of Bounded Natural Functors *} theory BNF_Axiomatization imports Main keywords "bnf_axiomatization" :: thy_decl begin ML_file "bnf_axiomatization.ML" end