src/HOL/Divides.thy
changeset 28562 4e74209f113e
parent 28262 aa7ca36d67fd
child 28823 dcbef866c9e2
--- a/src/HOL/Divides.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/Divides.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -127,7 +127,7 @@
   note that ultimately show thesis by blast
 qed
 
-lemma dvd_eq_mod_eq_0 [code func]: "a dvd b \<longleftrightarrow> b mod a = 0"
+lemma dvd_eq_mod_eq_0 [code]: "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
@@ -230,7 +230,7 @@
 begin
 
 definition divmod :: "nat \<Rightarrow> nat \<Rightarrow> nat \<times> nat" where
-  [code func del]: "divmod m n = (THE (q, r). divmod_rel m n q r)"
+  [code del]: "divmod m n = (THE (q, r). divmod_rel m n q r)"
 
 definition div_nat where
   "m div n = fst (divmod m n)"