Nominal/Ex/CPS/CPS3_DanvyFilinski.thy
changeset 2895 65efa1c7563c
parent 2882 186ec672cc51
child 2963 8b22497c25b9
equal deleted inserted replaced
2894:8ec94871de1e 2895:65efa1c7563c
     1 header {* CPS transformation of Danvy and Filinski *}
     1 header {* CPS transformation of Danvy and Filinski *}
     2 theory DanvyFilinski imports Lt begin
     2 theory CPS3_DanvyFilinski imports Lt begin
     3 
     3 
     4 nominal_primrec
     4 nominal_primrec
     5   CPS1 :: "lt \<Rightarrow> (lt \<Rightarrow> lt) \<Rightarrow> lt" ("_*_"  [100,100] 100)
     5   CPS1 :: "lt \<Rightarrow> (lt \<Rightarrow> lt) \<Rightarrow> lt" ("_*_"  [100,100] 100)
     6 and
     6 and
     7   CPS2 :: "lt \<Rightarrow> lt \<Rightarrow> lt" ("_^_" [100,100] 100)
     7   CPS2 :: "lt \<Rightarrow> lt \<Rightarrow> lt" ("_^_" [100,100] 100)