theory Term8imports "../NewParser"begin(* example 8 *)atom_decl nameML {* val _ = cheat_alpha_bn_rsp := true *}nominal_datatype foo = Foo0 "name"| Foo1 b::"bar" f::"foo" bind_set "bv b" in fand bar = Bar0 "name"| Bar1 "name" s::"name" b::"bar" bind_set s in bbinder bvwhere "bv (Bar0 x) = {}"| "bv (Bar1 v x b) = {atom v}"thm foo_bar.suppend