src/HOL/ex/Classpackage.thy
changeset 24348 c708ea5b109a
parent 24282 9b64aa297524
child 24423 ae9cd0e92423
equal deleted inserted replaced
24347:245ff8661b8c 24348:c708ea5b109a
   340 
   340 
   341 definition "x1 = X (1::nat) 2 3"
   341 definition "x1 = X (1::nat) 2 3"
   342 definition "x2 = X (1::int) 2 3"
   342 definition "x2 = X (1::int) 2 3"
   343 definition "y2 = Y (1::int) 2 3"
   343 definition "y2 = Y (1::int) 2 3"
   344 
   344 
   345 code_gen x1 x2 y2 in SML module_name Classpackage
   345 export_code x1 x2 y2 in SML module_name Classpackage
   346   in OCaml file -
   346   in OCaml file -
   347   in Haskell file -
   347   in Haskell file -
   348 
   348 
   349 end
   349 end