--- a/Nominal/Ex/TypeSchemes2.thy Mon May 19 11:19:48 2014 +0100
+++ b/Nominal/Ex/TypeSchemes2.thy Mon May 19 12:45:26 2014 +0100
@@ -61,7 +61,7 @@
using a
by clarsimp
-nominal_primrec (default "case_sum (\<lambda>x. Inl undefined) (\<lambda>x. Inr undefined)")
+nominal_function (default "case_sum (\<lambda>x. Inl undefined) (\<lambda>x. Inr undefined)")
subst :: "(name \<times> ty) list \<Rightarrow> ty \<Rightarrow> ty"
and substs :: "(name \<times> ty) list \<Rightarrow> tys \<Rightarrow> tys"
where