src/HOL/Trancl.thy
author clasohm
Tue, 30 Jan 1996 15:24:36 +0100
changeset 1465 5d7a7e439cec
parent 1301 42782316d510
child 1475 7f5a4cd08209
permissions -rw-r--r--
expanded tabs

(*  Title: 	HOL/Trancl.thy
    ID:         $Id$
    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1992  University of Cambridge

Relfexive and Transitive closure of a relation

rtrancl is refl&transitive closure;
trancl is transitive closure
reflcl is reflexive closure
*)

Trancl = Lfp + Relation + 
consts
    rtrancl :: "('a * 'a)set => ('a * 'a)set"	("(_^*)" [100] 100)
    trancl  :: "('a * 'a)set => ('a * 'a)set"	("(_^+)" [100] 100)  
syntax
    reflcl  :: "('a*'a)set => ('a*'a)set"       ("(_^=)" [100] 100)
defs   
  rtrancl_def	"r^*  ==  lfp(%s. id Un (r O s))"
  trancl_def	"r^+  ==  r O rtrancl(r)"
translations
                "r^=" == "r Un id"
end