src/HOL/Integ/IntPower.thy
author paulson
Mon, 05 Mar 2001 15:25:11 +0100
changeset 11193 851c90b23a9e
parent 9509 0f3ee1f89ca8
child 11701 3d51fbf81c17
permissions -rw-r--r--
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp

(*  Title:	IntPower.thy
    ID:         $Id$
    Author:	Thomas M. Rasmussen
    Copyright	2000  University of Cambridge

Integer powers 
*)

IntPower = IntDiv + 

instance
  int :: {power}

primrec
  power_0   "p ^ 0 = #1"
  power_Suc "p ^ (Suc n) = (p::int) * (p ^ n)"

end