codegen
authornipkow
Thu, 11 Dec 2008 08:56:02 +0100
changeset 29108 12ca66b887a0
parent 29107 e70b9c2bee14
child 29109 389ebed8b98e
codegen
src/HOL/Divides.thy
src/HOL/Real.thy
--- a/src/HOL/Divides.thy	Thu Dec 11 08:53:53 2008 +0100
+++ b/src/HOL/Divides.thy	Thu Dec 11 08:56:02 2008 +0100
@@ -127,7 +127,7 @@
   note that ultimately show thesis by blast
 qed
 
-lemma dvd_eq_mod_eq_0 [code]: "a dvd b \<longleftrightarrow> b mod a = 0"
+lemma dvd_eq_mod_eq_0 [code unfold]: "a dvd b \<longleftrightarrow> b mod a = 0"
 proof
   assume "b mod a = 0"
   with mod_div_equality [of b a] have "b div a * a = b" by simp
--- a/src/HOL/Real.thy	Thu Dec 11 08:53:53 2008 +0100
+++ b/src/HOL/Real.thy	Thu Dec 11 08:56:02 2008 +0100
@@ -1,5 +1,5 @@
 theory Real
-imports "~~/src/HOL/Real/RealVector"
+imports RComplete "~~/src/HOL/Real/RealVector"
 begin
 
 end