src/HOL/Divides.thy
changeset 29509 1ff0f3f08a7b
parent 29405 98ab21b14f09
child 29667 53103fc8ffa3
--- a/src/HOL/Divides.thy	Fri Jan 16 08:29:11 2009 +0100
+++ b/src/HOL/Divides.thy	Fri Jan 16 14:58:11 2009 +0100
@@ -20,7 +20,7 @@
 
 subsection {* Abstract division in commutative semirings. *}
 
-class semiring_div = comm_semiring_1_cancel + div + 
+class semiring_div = comm_semiring_1_cancel + div +
   assumes mod_div_equality: "a div b * b + a mod b = a"
     and div_by_0 [simp]: "a div 0 = 0"
     and div_0 [simp]: "0 div a = 0"
@@ -800,7 +800,7 @@
 
 text {* @{term "op dvd"} is a partial order *}
 
-class_interpretation dvd: order ["op dvd" "\<lambda>n m \<Colon> nat. n dvd m \<and> \<not> m dvd n"]
+interpretation dvd!: order "op dvd" "\<lambda>n m \<Colon> nat. n dvd m \<and> \<not> m dvd n"
   proof qed (auto intro: dvd_refl dvd_trans dvd_anti_sym)
 
 lemma dvd_diff: "[| k dvd m; k dvd n |] ==> k dvd (m-n :: nat)"