src/HOL/Nat.thy
changeset 58952 5d82cdef6c1b
parent 58889 5b7a9633cfa8
child 59000 6eb0725503fc
--- a/src/HOL/Nat.thy	Sat Nov 08 22:10:16 2014 +0100
+++ b/src/HOL/Nat.thy	Sat Nov 08 16:53:26 2014 +0100
@@ -785,9 +785,10 @@
   show "\<And>m n q :: nat. m < n \<Longrightarrow> 0 < q \<Longrightarrow> q * m < q * n" by (simp add: mult_less_mono2)
 qed
 
-instance nat :: no_zero_divisors
+instance nat :: semiring_no_zero_divisors
 proof
-  fix a::nat and b::nat show "a ~= 0 \<Longrightarrow> b ~= 0 \<Longrightarrow> a * b ~= 0" by auto
+  fix m n :: nat
+  show "m \<noteq> 0 \<Longrightarrow> n \<noteq> 0 \<Longrightarrow> m * n \<noteq> 0" by simp
 qed