src/HOL/ex/Codegenerator_Pretty.thy
changeset 24348 c708ea5b109a
parent 24249 1f60b45c5f97
child 24530 1bac25879117
equal deleted inserted replaced
24347:245ff8661b8c 24348:c708ea5b109a
    47   "R3' = real_of_rat (Fract 11 (-9))"
    47   "R3' = real_of_rat (Fract 11 (-9))"
    48 
    48 
    49 definition
    49 definition
    50   "foobar' = (foo' R1' 1 R3', bar' R2' 0 R3', foo' R1' R3' R2')"
    50   "foobar' = (foo' R1' 1 R3', bar' R2' 0 R3', foo' R1' R3' R2')"
    51 
    51 
    52 code_gen foobar foobar' in SML module_name Foo
    52 export_code foobar foobar' in SML module_name Foo
    53   in OCaml file -
    53   in OCaml file -
    54   in Haskell file -
    54   in Haskell file -
    55 ML {* (Foo.foobar, Foo.foobar') *}
    55 ML {* (Foo.foobar, Foo.foobar') *}
    56 
    56 
    57 end
    57 end