| author | wenzelm |
| Sat, 17 Sep 2005 12:18:04 +0200 | |
| changeset 17448 | b94e2897776a |
| parent 17278 | f27456a2a975 |
| child 19802 | c2860c37e574 |
| permissions | -rw-r--r-- |
(* Title: HOL/Hoare/Arith2.thy ID: $Id$ Author: Norbert Galm Copyright 1995 TUM More arithmetic. Much of this duplicates ex/Primes. *) theory Arith2 imports Main begin constdefs "cd" :: "[nat, nat, nat] => bool" "cd x m n == x dvd m & x dvd n" gcd :: "[nat, nat] => nat" "gcd m n == @x.(cd x m n) & (!y.(cd y m n) --> y<=x)" consts fac :: "nat => nat" primrec "fac 0 = Suc 0" "fac(Suc n) = (Suc n)*fac(n)" ML {* use_legacy_bindings (the_context ()) *} end