src/HOL/Extraction/QuotRem.thy
changeset 17145 e623e57b0f44
parent 16417 9bc16273c2d4
child 17604 5f30179fbf44
--- a/src/HOL/Extraction/QuotRem.thy	Thu Aug 25 16:10:16 2005 +0200
+++ b/src/HOL/Extraction/QuotRem.thy	Thu Aug 25 16:13:09 2005 +0200
@@ -6,7 +6,6 @@
 header {* Quotient and remainder *}
 
 theory QuotRem imports Main begin
-
 text {* Derivation of quotient and remainder using program extraction. *}
 
 lemma nat_eq_dec: "\<And>n::nat. m = n \<or> m \<noteq> n"
@@ -46,7 +45,8 @@
   @{thm [display] division_correctness [no_vars]}
 *}
 
-generate_code
+code_module Div
+contains
   test = "division 9 2"
 
 end