retain isolated blob nodes (amending deb2fcbda16e): avoid failure of Session.handle_change with "Missing blob", when opening theory with load command later;
(* 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