src/HOL/Integ/IntPower.thy
author skalberg
Fri, 29 Aug 2003 18:39:47 +0200
changeset 14176 716fec31f9ea
parent 11868 56db9f3a6b3e
child 14259 79f7d3451b1e
permissions -rw-r--r--
Added show_all_types flag, such that all type information in the term is made explicit.

(*  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