Lm1:
for a, b, c being Integer st a + 2 < b holds
((c - b) + 1) + 2 < (c - a) + 1
theorem Th7:
for
n being
odd Nat holds
( not
n <= 4 or
n = 1 or
n = 3 )
theorem Th8:
for
n being
odd Nat holds
( not
n <= 6 or
n = 1 or
n = 3 or
n = 5 )
theorem
for
n being
odd Nat holds
( not
n <= 8 or
n = 1 or
n = 3 or
n = 5 or
n = 7 )
theorem Th12:
for
n being
even Nat holds
( not
n <= 5 or
n = 0 or
n = 2 or
n = 4 )
theorem Th13:
for
n being
even Nat holds
( not
n <= 7 or
n = 0 or
n = 2 or
n = 4 or
n = 6 )
Lm2:
for i, j being odd Nat st i <= j holds
ex k being Nat st i + (2 * k) = j
scheme
FinGraphOrderCompInd{
P1[
set ] } :
provided
theorem Th46:
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
object st
(
P is
open &
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 )
Lm3:
for G being _Graph
for W being Walk of G st W is chordal holds
W .reverse() is chordal