src/HOL/Library/Primes.thy
changeset 21404 eb85850d3eb7
parent 21256 47195501ecf7
child 22665 cf152ff55d16
--- a/src/HOL/Library/Primes.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/Library/Primes.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -11,10 +11,11 @@
 begin
 
 definition
-  coprime :: "nat => nat => bool"
+  coprime :: "nat => nat => bool" where
   "coprime m n = (gcd (m, n) = 1)"
 
-  prime :: "nat \<Rightarrow> bool"
+definition
+  prime :: "nat \<Rightarrow> bool" where
   "prime p = (1 < p \<and> (\<forall>m. m dvd p --> m = 1 \<or> m = p))"