src/HOL/Extraction/QuotRem.thy
changeset 24348 c708ea5b109a
parent 23373 ead82c82da9e
child 25419 e6a56be0ccaa
--- a/src/HOL/Extraction/QuotRem.thy	Mon Aug 20 18:07:31 2007 +0200
+++ b/src/HOL/Extraction/QuotRem.thy	Mon Aug 20 18:07:49 2007 +0200
@@ -49,6 +49,6 @@
 contains
   test = "division 9 2"
 
-code_gen division in SML
+export_code division in SML
 
 end