|
10213
|
1 |
(* Title: HOL/Transitive_Closure.thy
|
|
|
2 |
ID: $Id$
|
|
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory
|
|
|
4 |
Copyright 1992 University of Cambridge
|
|
|
5 |
|
|
|
6 |
Relfexive and Transitive closure of a relation
|
|
|
7 |
|
|
|
8 |
rtrancl is reflexive/transitive closure;
|
|
|
9 |
trancl is transitive closure
|
|
|
10 |
reflcl is reflexive closure
|
|
|
11 |
|
|
10331
|
12 |
These postfix operators have MAXIMUM PRIORITY, forcing their operands
|
|
|
13 |
to be atomic.
|
|
10213
|
14 |
*)
|
|
|
15 |
|
|
10980
|
16 |
theory Transitive_Closure = Lfp + Relation
|
|
|
17 |
files ("Transitive_Closure_lemmas.ML"):
|
|
10213
|
18 |
|
|
|
19 |
constdefs
|
|
10331
|
20 |
rtrancl :: "('a * 'a) set => ('a * 'a) set" ("(_^*)" [1000] 999)
|
|
|
21 |
"r^* == lfp (%s. Id Un (r O s))"
|
|
10213
|
22 |
|
|
10331
|
23 |
trancl :: "('a * 'a) set => ('a * 'a) set" ("(_^+)" [1000] 999)
|
|
|
24 |
"r^+ == r O rtrancl r"
|
|
10213
|
25 |
|
|
|
26 |
syntax
|
|
10331
|
27 |
"_reflcl" :: "('a * 'a) set => ('a * 'a) set" ("(_^=)" [1000] 999)
|
|
10213
|
28 |
translations
|
|
|
29 |
"r^=" == "r Un Id"
|
|
|
30 |
|
|
10827
|
31 |
syntax (xsymbols)
|
|
10331
|
32 |
rtrancl :: "('a * 'a) set => ('a * 'a) set" ("(_\\<^sup>*)" [1000] 999)
|
|
|
33 |
trancl :: "('a * 'a) set => ('a * 'a) set" ("(_\\<^sup>+)" [1000] 999)
|
|
|
34 |
"_reflcl" :: "('a * 'a) set => ('a * 'a) set" ("(_\\<^sup>=)" [1000] 999)
|
|
|
35 |
|
|
10980
|
36 |
use "Transitive_Closure_lemmas.ML"
|
|
|
37 |
|
|
10213
|
38 |
end
|