Nominal/Ex/SFT/Consts.thy
changeset 3236 e2da10806a34
parent 3235 5ebd327ffb96
--- a/Nominal/Ex/SFT/Consts.thy	Mon May 19 12:45:26 2014 +0100
+++ b/Nominal/Ex/SFT/Consts.thy	Mon May 19 16:45:46 2014 +0100
@@ -99,7 +99,7 @@
     by (rule, perm_simp, rule)
 qed
 
-termination (eqvt) by lexicographic_order
+nominal_termination (eqvt) by lexicographic_order
 
 lemma supp_numeral[simp]:
   "supp \<lbrace>x\<rbrace> = supp x"
@@ -144,7 +144,7 @@
   apply (simp_all add: fresh_at_base lam.fresh eqvt_def eqvts_raw fresh_rev)
   done
 
-termination (eqvt) by lexicographic_order
+nominal_termination (eqvt) by lexicographic_order
 
 lemma ltgt_eq_iff[simp]:
   "\<guillemotleft>M\<guillemotright> = \<guillemotleft>N\<guillemotright> \<longleftrightarrow> M = N"