refined and added example for ExecutableRat
authorhaftmann
Tue, 16 Jan 2007 08:12:09 +0100
changeset 22071 ebcfe7c2499d
parent 22070 a10ad9d71eaf
child 22072 aabbf8c4de80
refined and added example for ExecutableRat
src/HOL/ex/Codegenerator_Rat.thy
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/ex/Codegenerator_Rat.thy	Tue Jan 16 08:12:09 2007 +0100
@@ -0,0 +1,39 @@
+(*  Title:      HOL/Library/ExecutableRat.thy
+    ID:         $Id$
+    Author:     Florian Haftmann, TU Muenchen
+*)
+
+header {* Simple example for executable rational numbers *}
+
+theory Codegenerator_Rat
+imports ExecutableRat EfficientNat
+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 (SML #) (SML -)
+ML {* ROOT.Codegenerator_Rat.foobar *}
+
+code_module Foo
+  contains foobar
+ML {* Foo.foobar *}
+
+end