Nominal/Ex/CPS/CPS3_DanvyFilinski.thy
changeset 3235 5ebd327ffb96
parent 3231 188826f1ccdb
child 3245 017e33849f4d
--- a/Nominal/Ex/CPS/CPS3_DanvyFilinski.thy	Mon May 19 11:19:48 2014 +0100
+++ b/Nominal/Ex/CPS/CPS3_DanvyFilinski.thy	Mon May 19 12:45:26 2014 +0100
@@ -1,7 +1,7 @@
 header {* CPS transformation of Danvy and Filinski *}
 theory CPS3_DanvyFilinski imports Lt begin
 
-nominal_primrec
+nominal_function
   CPS1 :: "lt \<Rightarrow> (lt \<Rightarrow> lt) \<Rightarrow> lt" ("_*_"  [100,100] 100)
 and
   CPS2 :: "lt \<Rightarrow> lt \<Rightarrow> lt" ("_^_" [100,100] 100)