Nominal/Ex/Beta.thy
changeset 3235 5ebd327ffb96
parent 3077 df1055004f52
child 3236 e2da10806a34
--- a/Nominal/Ex/Beta.thy	Mon May 19 11:19:48 2014 +0100
+++ b/Nominal/Ex/Beta.thy	Mon May 19 12:45:26 2014 +0100
@@ -14,7 +14,7 @@
 
 section {* capture-avoiding substitution *}
 
-nominal_primrec
+nominal_function
   subst :: "lam \<Rightarrow> name \<Rightarrow> lam \<Rightarrow> lam"  ("_ [_ ::= _]" [90, 90, 90] 90)
 where
   "(Var x)[y ::= s] = (if x = y then s else (Var x))"