src/HOL/Hoare/Arith2.thy
changeset 35416 d8d7d1b785af
parent 33657 a4179bf442d1
child 38353 d98baa2cf589
--- a/src/HOL/Hoare/Arith2.thy	Wed Feb 24 11:55:52 2010 +0100
+++ b/src/HOL/Hoare/Arith2.thy	Mon Mar 01 13:40:23 2010 +0100
@@ -1,5 +1,4 @@
 (*  Title:      HOL/Hoare/Arith2.thy
-    ID:         $Id$
     Author:     Norbert Galm
     Copyright   1995 TUM
 
@@ -10,11 +9,10 @@
 imports Main
 begin
 
-constdefs
-  "cd"    :: "[nat, nat, nat] => bool"
+definition "cd" :: "[nat, nat, nat] => bool" where
   "cd x m n  == x dvd m & x dvd n"
 
-  gcd     :: "[nat, nat] => nat"
+definition gcd     :: "[nat, nat] => nat" where
   "gcd m n     == @x.(cd x m n) & (!y.(cd y m n) --> y<=x)"
 
 consts fac     :: "nat => nat"