moved the exporting part into the parser (this is still a hack); re-added CoreHaskell again to the examples - there seems to be a problem with the variable name pat
theory Ex1recimports "../NewParser"beginatom_decl nameML {* val _ = cheat_supp_eq := true *}ML {* val _ = cheat_equivp := true *}nominal_datatype lam = Var "name"| App "lam" "lam"| Lam x::"name" t::"lam" bind_set x in t| Let bp::"bp" t::"lam" bind_set "bi bp" in bp tand bp = Bp "name" "lam"binder bi::"bp \<Rightarrow> atom set"where "bi (Bp x t) = {atom x}"thm lam_bp.fvthm lam_bp.eq_iff[no_vars]thm lam_bp.bnthm lam_bp.permthm lam_bp.inductthm lam_bp.inductsthm lam_bp.distinctthm lam_bp.suppML {* Sign.of_sort @{theory} (@{typ lam}, @{sort fs}) *}thm lam_bp.fv[simplified lam_bp.supp(1-2)]end