1
(* Title: HOL/RelPow.thy
2
ID: $Id$
3
Author: Tobias Nipkow
4
Copyright 1996 TU Muenchen
5
6
R^n = R O ... O R, the n-fold composition of R
7
*)
8
9
RelPow = Nat +
10
11
primrec "op ^" nat
12
"R^0 = id"
13
"R^(Suc n) = R O (R^n)"
14
15
end