Lm1:
for F being Function
for x, y being set holds dom (F +* (x .--> y)) = (dom F) \/ {x}
Lm2:
for f being one-to-one Function
for X, Y being set st X c= Y holds
for x being set st x in dom ((f | X) ") holds
((f | X) ") . x = ((f | Y) ") . x
Lm3:
for a, b, c being Real st a < b holds
(c - b) + 1 < (c - a) + 1
theorem Th2:
for
n,
m,
k being
Nat st
m <= k &
n < m holds
k -' m < k -' n
Lm4:
for G being _Graph
for W being Walk of G
for e, v being object st e Joins W .last() ,v,G holds
(W .addEdge e) .length() = (W .length()) + 1
Lm5:
for G being _Graph
for W being Walk of G holds W .length() = (W .reverse()) .length()
Lm6:
for G being _Graph
for W being Walk of G
for e, x being object st e Joins W .last() ,x,G holds
for n being Nat st n in dom W holds
( (W .addEdge e) . n = W . n & n in dom (W .addEdge e) )
definition
let G be
_finite _Graph;
let L be
LexBFS:Labeling of
G;
existence
( ( dom (L `1) = the_Vertices_of G implies ex b1 being Vertex of G st b1 = the Element of the_Vertices_of G ) & ( not dom (L `1) = the_Vertices_of G implies ex b1 being Vertex of G ex S being non empty finite Subset of (bool NAT) ex B being non empty finite Subset of (Bags NAT) ex F being Function st
( S = rng F & F = (L `2) | ((the_Vertices_of G) \ (dom (L `1))) & ( for x being finite Subset of NAT st x in S holds
(x,1) -bag in B ) & ( for x being set st x in B holds
ex y being finite Subset of NAT st
( y in S & x = (y,1) -bag ) ) & b1 = the Element of F " {(support (max (B,(InvLexOrder NAT))))} ) ) )
uniqueness
for b1, b2 being Vertex of G holds
( ( dom (L `1) = the_Vertices_of G & b1 = the Element of the_Vertices_of G & b2 = the Element of the_Vertices_of G implies b1 = b2 ) & ( not dom (L `1) = the_Vertices_of G & ex S being non empty finite Subset of (bool NAT) ex B being non empty finite Subset of (Bags NAT) ex F being Function st
( S = rng F & F = (L `2) | ((the_Vertices_of G) \ (dom (L `1))) & ( for x being finite Subset of NAT st x in S holds
(x,1) -bag in B ) & ( for x being set st x in B holds
ex y being finite Subset of NAT st
( y in S & x = (y,1) -bag ) ) & b1 = the Element of F " {(support (max (B,(InvLexOrder NAT))))} ) & ex S being non empty finite Subset of (bool NAT) ex B being non empty finite Subset of (Bags NAT) ex F being Function st
( S = rng F & F = (L `2) | ((the_Vertices_of G) \ (dom (L `1))) & ( for x being finite Subset of NAT st x in S holds
(x,1) -bag in B ) & ( for x being set st x in B holds
ex y being finite Subset of NAT st
( y in S & x = (y,1) -bag ) ) & b2 = the Element of F " {(support (max (B,(InvLexOrder NAT))))} ) implies b1 = b2 ) )
consistency
for b1 being Vertex of G holds verum
;
end;