| author | wenzelm |
| Tue, 23 Oct 2001 22:52:31 +0200 | |
| changeset 11908 | 82f68fd05094 |
| parent 11701 | 3d51fbf81c17 |
| child 12018 | ec054019c910 |
| permissions | -rw-r--r-- |
(* Title : HOL/Real/RealPow.thy ID : $Id$ Author : Jacques D. Fleuriot Copyright : 1998 University of Cambridge Description : Natural powers theory *) theory RealPow = RealAbs: (*belongs to theory RealAbs*) lemmas [arith_split] = abs_split instance real :: power .. primrec (realpow) realpow_0: "r ^ 0 = Numeral1" realpow_Suc: "r ^ (Suc n) = (r::real) * (r ^ n)" end