corrected code generator module names
authorhaftmann
Fri, 10 Aug 2007 17:10:04 +0200
changeset 24223 fa9421d52c74
parent 24222 a8a28c15c5cc
child 24224 a5c95bbeb31d
corrected code generator module names
src/HOL/Library/Executable_Rat.thy
--- a/src/HOL/Library/Executable_Rat.thy	Fri Aug 10 17:10:03 2007 +0200
+++ b/src/HOL/Library/Executable_Rat.thy	Fri Aug 10 17:10:04 2007 +0200
@@ -94,12 +94,15 @@
   unfolding Rat_def by simp
 
 code_modulename SML
+  Rational Rational
   Executable_Rat Rational
 
 code_modulename OCaml
+  Rational Rational
   Executable_Rat Rational
 
 code_modulename Haskell
+  Rational Rational
   Executable_Rat Rational
 
 end