set SA0 = Start-At (0,SCM+FSA);
set Q = (intloc 0) .--> 1;
theorem Th8:
for
P1,
P2 being
Instruction-Sequence of
SCM+FSA for
s1 being
0 -started State of
SCM+FSA for
s2 being
State of
SCM+FSA for
I being
really-closed Program of
SCM+FSA st
I c= P1 holds
for
n being
Nat st
Reloc (
I,
n)
c= P2 &
IC s2 = n &
DataPart s1 = DataPart s2 holds
for
i being
Nat holds
(
(IC (Comput (P1,s1,i))) + n = IC (Comput (P2,s2,i)) &
IncAddr (
(CurInstr (P1,(Comput (P1,s1,i)))),
n)
= CurInstr (
P2,
(Comput (P2,s2,i))) &
DataPart (Comput (P1,s1,i)) = DataPart (Comput (P2,s2,i)) )
theorem Th9:
for
P1,
P2 being
Instruction-Sequence of
SCM+FSA for
s1,
s2 being
0 -started State of
SCM+FSA for
I being
really-closed Program of
SCM+FSA st
I c= P1 &
I c= P2 &
DataPart s1 = DataPart s2 holds
for
i being
Nat holds
(
IC (Comput (P1,s1,i)) = IC (Comput (P2,s2,i)) &
CurInstr (
P1,
(Comput (P1,s1,i)))
= CurInstr (
P2,
(Comput (P2,s2,i))) &
DataPart (Comput (P1,s1,i)) = DataPart (Comput (P2,s2,i)) )
theorem Th14:
for
P1,
P2 being
Instruction-Sequence of
SCM+FSA for
s1 being
0 -started State of
SCM+FSA for
s2 being
State of
SCM+FSA for
I being
Program of
SCM+FSA st
I c= P1 &
I is_pseudo-closed_on s1,
P1 holds
for
n being
Nat st
Reloc (
I,
n)
c= P2 &
IC s2 = n &
DataPart s1 = DataPart s2 holds
( ( for
i being
Nat st
i < pseudo-LifeSpan (
s1,
P1,
I) holds
IncAddr (
(CurInstr (P1,(Comput (P1,s1,i)))),
n)
= CurInstr (
P2,
(Comput (P2,s2,i))) ) & ( for
i being
Nat st
i <= pseudo-LifeSpan (
s1,
P1,
I) holds
(
(IC (Comput (P1,s1,i))) + n = IC (Comput (P2,s2,i)) &
DataPart (Comput (P1,s1,i)) = DataPart (Comput (P2,s2,i)) ) ) )
theorem Th21:
for
P being
Instruction-Sequence of
SCM+FSA for
s being
State of
SCM+FSA for
I being
Program of
SCM+FSA st
Directed I is_pseudo-closed_on s,
P holds
(
I ";" (Stop SCM+FSA) is_halting_on s,
P &
LifeSpan (
(P +* (I ";" (Stop SCM+FSA))),
(Initialize s))
= pseudo-LifeSpan (
s,
P,
(Directed I)) & ( for
n being
Nat st
n < pseudo-LifeSpan (
s,
P,
(Directed I)) holds
IC (Comput ((P +* I),(Initialize s),n)) = IC (Comput ((P +* (I ";" (Stop SCM+FSA))),(Initialize s),n)) ) & ( for
n being
Nat st
n <= pseudo-LifeSpan (
s,
P,
(Directed I)) holds
DataPart (Comput ((P +* I),(Initialize s),n)) = DataPart (Comput ((P +* (I ";" (Stop SCM+FSA))),(Initialize s),n)) ) )
theorem Th34:
for
P being
Instruction-Sequence of
SCM+FSA for
s being
State of
SCM+FSA for
I,
J being
MacroInstruction of
SCM+FSA for
a being
read-write Int-Location st
s . a <= 0 &
Directed J is_pseudo-closed_on s,
P holds
(
if>0 (
a,
I,
J)
is_halting_on s,
P &
LifeSpan (
(P +* (if>0 (a,I,J))),
(s +* (Start-At (0,SCM+FSA))))
= (LifeSpan ((P +* (J ";" (Stop SCM+FSA))),(Initialize s))) + 3 )
theorem Th49:
for
P being
Instruction-Sequence of
SCM+FSA for
s being
State of
SCM+FSA for
I being
Program of
SCM+FSA st
I is_halting_on Initialized s,
P holds
( ( for
a being
read-write Int-Location holds
(IExec (I,P,s)) . a = (Comput ((P +* I),(Initialize (Initialized s)),(LifeSpan ((P +* I),(Initialize (Initialized s)))))) . a ) & ( for
f being
FinSeq-Location holds
(IExec (I,P,s)) . f = (Comput ((P +* I),(Initialize (Initialized s)),(LifeSpan ((P +* I),(Initialize (Initialized s)))))) . f ) )
theorem Th62:
for
P1,
P2 being
Instruction-Sequence of
SCM+FSA for
s1,
s2 being
State of
SCM+FSA for
I being
really-closed Program of
SCM+FSA st
I is_halting_on s1,
P1 &
DataPart s1 = DataPart s2 holds
for
k being
Nat holds
(
Comput (
(P1 +* I),
(Initialize s1),
k)
= Comput (
(P2 +* I),
(Initialize s2),
k) &
CurInstr (
(P1 +* I),
(Comput ((P1 +* I),(Initialize s1),k)))
= CurInstr (
(P2 +* I),
(Comput ((P2 +* I),(Initialize s2),k))) )
canceled;
Lm1:
for aa being Int-Location
for I, J being MacroInstruction of SCM+FSA st not I destroys aa & not J destroys aa holds
not I ';' J destroys aa
Lm2:
for aa being Int-Location
for I being MacroInstruction of SCM+FSA st not I destroys aa holds
not I ';' (goto 0) destroys aa
Lm3:
for aa, bb being Int-Location
for I being MacroInstruction of SCM+FSA st not I destroys aa holds
not if>0 (bb,(I ';' (goto 0))) destroys aa