(* Title: N2M Authors: Jasmin Blanchette, Andrei Popescu, Dmitriy Traytel Maintainer: Dmitriy Traytel <traytel at inf.ethz.ch> *) section ‹Mutual View on Nested Datatypes› (*<*) theory N2M imports "HOL-Library.BNF_Axiomatization" begin (*>*) notation BNF_Def.convol (‹<_, _>›) declare [[bnf_internals]] declare [[typedef_overloaded]] bnf_axiomatization ('a, 'b) F0 [wits: "'a ⇒ ('a, 'b) F0"] bnf_axiomatization ('a, 'b) G0 [wits: "'a ⇒ ('a, 'b) G0"] subsection ‹Nested Definition›