changeset 37826 | 4c0a5e35931a |
parent 37765 | 26bdfb7b680b |
child 38054 | acd48ef85bfc |
--- a/src/HOL/ex/Numeral.thy Wed Jul 14 16:02:50 2010 +0200 +++ b/src/HOL/ex/Numeral.thy Wed Jul 14 16:13:14 2010 +0200 @@ -988,9 +988,9 @@ subsection {* Toy examples *} definition "bar \<longleftrightarrow> #4 * #2 + #7 = (#8 :: nat) \<and> #4 * #2 + #7 \<ge> (#8 :: int) - #3" + code_thms bar -export_code bar in Haskell file - -export_code bar in OCaml module_name Foo file - -ML {* @{code bar} *} + +export_code bar checking SML OCaml? Haskell? end