src/HOL/BNF/Examples/Misc_Codata.thy
changeset 49617 7ec6471f8388
parent 49591 91b228e26348
child 51804 be6e703908f4
--- a/src/HOL/BNF/Examples/Misc_Codata.thy	Thu Sep 27 12:08:38 2012 +0200
+++ b/src/HOL/BNF/Examples/Misc_Codata.thy	Thu Sep 27 17:00:54 2012 +0200
@@ -58,11 +58,15 @@
    and ('a, 'b, 'c) in_here =
   IH1 'b 'a | IH2 'c
 
-codata_raw some_killing': 'a = "'b \<Rightarrow> 'd \<Rightarrow> ('a + 'c)"
-and in_here': 'c = "'d + 'e"
+codata ('a, 'b, 'c) some_killing' =
+  SK' "'a \<Rightarrow> 'b \<Rightarrow> ('a, 'b, 'c) some_killing' + ('a, 'b, 'c) in_here'"
+   and ('a, 'b, 'c) in_here' =
+  IH1' 'b | IH2' 'c
 
-codata_raw some_killing'': 'a = "'b \<Rightarrow> 'c"
-and in_here'': 'c = "'d \<times> 'b + 'e"
+codata ('a, 'b, 'c) some_killing'' =
+  SK'' "'a \<Rightarrow> ('a, 'b, 'c) in_here''"
+   and ('a, 'b, 'c) in_here'' =
+  IH1'' 'b 'a | IH2'' 'c
 
 codata ('b, 'c) less_killing = LK "'b \<Rightarrow> 'c"