Nominal/Ex/CPS/CPS3_DanvyFilinski.thy
changeset 2895 65efa1c7563c
parent 2882 186ec672cc51
child 2963 8b22497c25b9
--- a/Nominal/Ex/CPS/CPS3_DanvyFilinski.thy	Fri Jun 24 10:54:31 2011 +0900
+++ b/Nominal/Ex/CPS/CPS3_DanvyFilinski.thy	Fri Jun 24 11:03:53 2011 +0900
@@ -1,5 +1,5 @@
 header {* CPS transformation of Danvy and Filinski *}
-theory DanvyFilinski imports Lt begin
+theory CPS3_DanvyFilinski imports Lt begin
 
 nominal_primrec
   CPS1 :: "lt \<Rightarrow> (lt \<Rightarrow> lt) \<Rightarrow> lt" ("_*_"  [100,100] 100)