src/HOL/ex/Codegenerator_Rat.thy
changeset 24203 a365995c043b
parent 24202 9e77397eba8e
child 24204 92c646714237
--- a/src/HOL/ex/Codegenerator_Rat.thy	Thu Aug 09 15:52:57 2007 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,41 +0,0 @@
-(*  Title:      HOL/Library/ExecutableRat.thy
-    ID:         $Id$
-    Author:     Florian Haftmann, TU Muenchen
-*)
-
-header {* Simple example for executable rational numbers *}
-
-theory Codegenerator_Rat
-imports Executable_Rat Efficient_Nat
-begin
-
-definition
-  foo :: "rat \<Rightarrow> rat \<Rightarrow> rat \<Rightarrow> rat" where
-  "foo r s t = (t + s) / t"
-
-definition
-  bar :: "rat \<Rightarrow> rat \<Rightarrow> rat \<Rightarrow> bool" where
-  "bar r s t \<longleftrightarrow> (r - s) \<le> t \<or> (s - t) \<le> r"
-
-definition
-  "R1 = Fract 3 7"
-
-definition
-  "R2 = Fract (-7) 5"
-
-definition
-  "R3 = Fract 11 (-9)"
-
-definition
-  "foobar = (foo R1 1 R3, bar R2 0 R3, foo R1 R3 R2)"
-
-code_gen foobar in SML to Foo
-  in OCaml file -
-  in Haskell file -
-ML {* Foo.foobar *}
-
-code_module Foo
-  contains foobar
-ML {* Foo.foobar *}
-
-end