begin
theorem Th1:
theorem Th2:
Lm1:
for a, b, c being Integer st a + 2 < b holds
((c - b) + 1) + 2 < (c - a) + 1
theorem Th3:
theorem Th4:
theorem Th5:
theorem Th6:
theorem Th7:
theorem Th8:
theorem
theorem Th10:
theorem Th11:
theorem Th12:
theorem Th13:
Lm2:
for i, j being natural odd number st i <= j holds
ex k being natural number st i + (2 * k) = j
theorem
theorem Th15:
:: deftheorem defines .followSet CHORD:def 1 :
for p being FinSequence
for n being natural number holds p .followSet n = rng ((n,(len p)) -cut p);
theorem Th16:
theorem Th17:
theorem Th18:
begin
theorem Th19:
theorem
theorem Th21:
theorem Th22:
theorem Th23:
theorem Th24:
theorem Th25:
theorem
theorem Th27:
theorem Th28:
theorem Th29:
theorem Th30:
theorem Th31:
scheme
FinGraphOrderCompInd{
P1[
set ] } :
provided
theorem Th32:
theorem Th33:
begin
:: deftheorem Def2 defines minlength CHORD:def 2 :
for G being _Graph
for W being Walk of G holds
( W is minlength iff for W2 being Walk of G st W2 is_Walk_from W .first() ,W .last() holds
len W2 >= len W );
theorem Th34:
theorem Th35:
theorem
theorem
theorem Th38:
theorem Th39:
theorem Th40:
theorem Th41:
theorem Th42:
theorem
begin
:: deftheorem Def3 defines are_adjacent CHORD:def 3 :
for G being _Graph
for a, b being Vertex of G holds
( a,b are_adjacent iff ex e being set st e Joins a,b,G );
theorem Th44:
theorem Th45:
theorem Th46:
theorem Th47:
for
G being
_Graph for
v1,
v2,
v3 being
Vertex of
G st
v1 <> v2 &
v1 <> v3 &
v2 <> v3 &
v1,
v2 are_adjacent &
v2,
v3 are_adjacent holds
ex
P being
Path of
G ex
e1,
e2 being
set st
( not
P is
closed &
len P = 5 &
P .length() = 2 &
e1 Joins v1,
v2,
G &
e2 Joins v2,
v3,
G &
P .edges() = {e1,e2} &
P .vertices() = {v1,v2,v3} &
P . 1
= v1 &
P . 3
= v2 &
P . 5
= v3 )
theorem Th48:
:: deftheorem defines .AdjacentSet CHORD:def 4 :
for G being _Graph
for S being set holds G .AdjacentSet S = { u where u is Vertex of G : ( not u in S & ex v being Vertex of G st
( v in S & u,v are_adjacent ) ) } ;
theorem
theorem Th50:
theorem Th51:
theorem Th52:
theorem
theorem
theorem Th55:
theorem
theorem Th57:
theorem Th58:
:: deftheorem Def5 defines AdjGraph CHORD:def 5 :
for G being _Graph
for S being set
for b3 being Subgraph of G st S is Subset of (the_Vertices_of G) holds
( b3 is AdjGraph of G,S iff b3 is inducedSubgraph of G,(G .AdjacentSet S) );
theorem Th59:
theorem Th60:
:: deftheorem Def6 defines complete CHORD:def 6 :
for G being _Graph holds
( G is complete iff for u, v being Vertex of G st u <> v holds
u,v are_adjacent );
theorem Th61:
theorem Th62:
theorem Th63:
begin
:: deftheorem Def7 defines simplicial CHORD:def 7 :
for G being _Graph
for v being Vertex of G holds
( v is simplicial iff ( G .AdjacentSet {v} <> {} implies for G2 being AdjGraph of G,{v} holds G2 is complete ) );
theorem Th64:
theorem Th65:
theorem Th66:
theorem Th67:
theorem Th68:
theorem Th69:
begin
:: deftheorem Def8 defines VertexSeparator CHORD:def 8 :
for G being _Graph
for a, b being Vertex of G st a <> b & not a,b are_adjacent holds
for b4 being Subset of (the_Vertices_of G) holds
( b4 is VertexSeparator of a,b iff ( not a in b4 & not b in b4 & ( for G2 being removeVertices of G,b4
for W being Walk of G2 holds not W is_Walk_from a,b ) ) );
theorem Th70:
theorem Th71:
theorem Th72:
theorem Th73:
theorem
theorem Th75:
theorem Th76:
theorem Th77:
:: deftheorem Def9 defines minimal CHORD:def 9 :
for G being _Graph
for a, b being Vertex of G
for S being VertexSeparator of a,b holds
( S is minimal iff for T being Subset of S st T <> S holds
not T is VertexSeparator of a,b );
theorem
theorem Th79:
theorem Th80:
theorem
theorem Th82:
theorem Th83:
begin
:: deftheorem Def10 defines chordal CHORD:def 10 :
for G being _Graph
for W being Walk of G holds
( W is chordal iff ex m, n being natural odd number st
( m + 2 < n & n <= len W & W . m <> W . n & ex e being set st e Joins W . m,W . n,G & ( for f being set st f in W .edges() holds
not f Joins W . m,W . n,G ) ) );
theorem Th84:
theorem Th85:
theorem Th86:
theorem Th87:
theorem
theorem Th89:
theorem
Lm3:
for G being _Graph
for W being Walk of G st W is chordal holds
W .reverse() is chordal
theorem
theorem Th92:
theorem
theorem
:: deftheorem Def11 defines chordal CHORD:def 11 :
for G being _Graph holds
( G is chordal iff for P being Walk of G st P .length() > 3 & P is Cycle-like holds
P is chordal );
theorem Th95:
theorem Th96:
theorem
theorem Th98:
theorem
theorem Th100:
theorem
theorem Th102:
theorem Th103:
begin
:: deftheorem Def12 defines VertexScheme CHORD:def 12 :
for G being finite _Graph
for b2 being FinSequence of the_Vertices_of G holds
( b2 is VertexScheme of G iff ( b2 is one-to-one & rng b2 = the_Vertices_of G ) );
theorem
theorem
theorem Th106:
theorem Th107:
:: deftheorem Def13 defines perfect CHORD:def 13 :
for G being finite _Graph
for S being VertexScheme of G holds
( S is perfect iff for n being non zero natural number st n <= len S holds
for Gf being inducedSubgraph of G,(S .followSet n)
for v being Vertex of Gf st v = S . n holds
v is simplicial );
theorem Th108:
theorem
theorem
theorem