changeset 35416 | d8d7d1b785af |
parent 33750 | 0a0d6d79d984 |
child 36745 | 403585a89772 |
--- a/doc-src/TutorialI/Rules/Primes.thy Wed Feb 24 11:55:52 2010 +0100 +++ b/doc-src/TutorialI/Rules/Primes.thy Mon Mar 01 13:40:23 2010 +0100 @@ -99,8 +99,7 @@ (**** The material below was omitted from the book ****) -constdefs - is_gcd :: "[nat,nat,nat] \<Rightarrow> bool" (*gcd as a relation*) +definition is_gcd :: "[nat,nat,nat] \<Rightarrow> bool" where (*gcd as a relation*) "is_gcd p m n == p dvd m \<and> p dvd n \<and> (ALL d. d dvd m \<and> d dvd n \<longrightarrow> d dvd p)"