author | wenzelm |
Thu, 13 Feb 2025 16:36:57 +0100 | |
changeset 82159 | f3a5a7c64412 |
parent 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 \<open>../Tools/BNF/bnf_axiomatization.ML\<close> end