small adjustments
authorhaftmann
Sun, 23 Jul 2006 07:21:41 +0200
changeset 20187 af47971ea304
parent 20186 56207a6f4cc5
child 20188 8b22026445af
small adjustments
src/HOL/ex/Classpackage.thy
src/HOL/ex/Codegenerator.thy
--- a/src/HOL/ex/Classpackage.thy	Sun Jul 23 07:21:22 2006 +0200
+++ b/src/HOL/ex/Classpackage.thy	Sun Jul 23 07:21:41 2006 +0200
@@ -312,7 +312,6 @@
 code_generate (ml, haskell) x
 code_generate (ml, haskell) y
 
-code_serialize ml (_)
 code_serialize ml (-)
 
 end
--- a/src/HOL/ex/Codegenerator.thy	Sun Jul 23 07:21:22 2006 +0200
+++ b/src/HOL/ex/Codegenerator.thy	Sun Jul 23 07:21:41 2006 +0200
@@ -2,7 +2,7 @@
     Author:     Florian Haftmann, TU Muenchen
 *)
 
-header {* Test and Examples for Code Generator *}
+header {* Test and Examples for code generator *}
 
 theory Codegenerator
 imports Main
@@ -46,6 +46,8 @@
 
 code_generate (ml, haskell) Pair fst snd Let split swap swapp appl
 
+subsection {* integers *}
+
 definition
   k :: "int"
   "k = 42"
@@ -64,6 +66,8 @@
   "op < :: int \<Rightarrow> int \<Rightarrow> bool"
   "op <= :: int \<Rightarrow> int \<Rightarrow> bool"
   fac
+  "op div :: int \<Rightarrow> int \<Rightarrow> int"
+  "op mod :: int \<Rightarrow> int \<Rightarrow> int"  
 
 subsection {* sums *}