src/HOL/Codatatype/Examples/Misc_Data.thy
changeset 49436 37cae324d73e
parent 49219 c28dd8326f9a
child 49456 fa8302c8dea1
equal deleted inserted replaced
49435:483007ddbdc2 49436:37cae324d73e
   143  and s6 = S61 s6 | S62 s1 s2 | S63 s6
   143  and s6 = S61 s6 | S62 s1 s2 | S63 s6
   144  and s7 = S71 s8 | S72 s5
   144  and s7 = S71 s8 | S72 s5
   145  and s8 = S8 nat
   145  and s8 = S8 nat
   146 *)
   146 *)
   147 
   147 
   148 data ('a, 'b) bar = BAR "'b \<Rightarrow> 'a"
   148 data ('a, 'b) bar = Bar "'b \<Rightarrow> 'a"
   149 data ('a, 'b, 'c, 'd) foo = FOO "'d + 'b \<Rightarrow> 'c + 'a"
   149 data ('a, 'b, 'c, 'd) foo = Foo "'d + 'b \<Rightarrow> 'c + 'a"
   150 
   150 
   151 data 'a dead_foo = A
   151 data 'a dead_foo = A
   152 data ('a, 'b) use_dead_foo = Y "'a" "'b dead_foo"
   152 data ('a, 'b) use_dead_foo = Y "'a" "'b dead_foo"
   153 
   153 
   154 end
   154 end