| author | wenzelm |
| Wed, 10 Jun 2015 21:49:02 +0200 | |
| changeset 60422 | be7565a1115b |
| parent 59794 | 39442248a027 |
| child 60500 | 903bb1495239 |
| 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