--- a/Nominal/Ex/LetRecFunNo.thy Mon May 19 12:45:26 2014 +0100
+++ b/Nominal/Ex/LetRecFunNo.thy Mon May 19 16:45:46 2014 +0100
@@ -53,7 +53,7 @@
apply clarify
apply metis
done
-termination (eqvt) by lexicographic_order
+nominal_termination (eqvt) by lexicographic_order
nominal_function substarec :: "(name \<Rightarrow> trm \<Rightarrow> assn \<Rightarrow> assn) \<Rightarrow> assn \<Rightarrow> assn" where
"substarec fac ANil = ANil"
@@ -64,7 +64,7 @@
apply (rule_tac y="b" in trm_assn.exhaust(2))
apply auto
done
-termination (eqvt) by lexicographic_order
+nominal_termination (eqvt) by lexicographic_order
lemma [fundef_cong]:
"(\<And>t1 t2. t = App t1 t2 \<Longrightarrow> fa t1 t2 = fa' t1 t2) \<Longrightarrow>