set D = Data-Locations ;
set SAt = Start-At (0,SCM+FSA);
Lm1:
for p being Instruction-Sequence of SCM+FSA
for I being good really-closed Program of SCM+FSA
for J being really-closed Program of SCM+FSA
for s being State of SCM+FSA st s . (intloc 0) = 1 & I is_halting_on s,p & J is_halting_on IExec (I,p,s),p & Initialize ((intloc 0) .--> 1) c= s & I ";" J c= p holds
( IC (Comput (p,s,((LifeSpan ((p +* I),s)) + 1))) = card I & DataPart (Comput (p,s,((LifeSpan ((p +* I),s)) + 1))) = DataPart (Initialized (Comput ((p +* I),s,(LifeSpan ((p +* I),s))))) & Reloc (J,(card I)) c= p & (Comput (p,s,((LifeSpan ((p +* I),s)) + 1))) . (intloc 0) = 1 & p halts_on s & LifeSpan (p,s) = ((LifeSpan ((p +* I),s)) + 1) + (LifeSpan (((p +* I) +* J),(Initialized (Result ((p +* I),s))))) & ( J is good implies (Result (p,s)) . (intloc 0) = 1 ) )
theorem Th5:
for
p being
Instruction-Sequence of
SCM+FSA for
s being
State of
SCM+FSA for
Ig being
good really-closed Program of
SCM+FSA for
J being
really-closed Program of
SCM+FSA st
Ig is_halting_on Initialized s,
p &
J is_halting_on IExec (
Ig,
p,
s),
p holds
IExec (
(Ig ";" J),
p,
s)
= (IExec (J,p,(IExec (Ig,p,s)))) +* (Start-At (((IC (IExec (J,p,(IExec (Ig,p,s))))) + (card Ig)),SCM+FSA))
theorem Th6:
for
p being
Instruction-Sequence of
SCM+FSA for
s being
State of
SCM+FSA for
a being
Int-Location for
Ig being
good really-closed Program of
SCM+FSA for
J being
really-closed Program of
SCM+FSA st (
Ig is
parahalting or
Ig is_halting_on Initialized s,
p ) & (
J is
parahalting or
J is_halting_on IExec (
Ig,
p,
s),
p ) holds
(IExec ((Ig ";" J),p,s)) . a = (IExec (J,p,(IExec (Ig,p,s)))) . a
theorem Th7:
for
p being
Instruction-Sequence of
SCM+FSA for
s being
State of
SCM+FSA for
f being
FinSeq-Location for
Ig being
good really-closed Program of
SCM+FSA for
J being
really-closed Program of
SCM+FSA st (
Ig is
parahalting or
Ig is_halting_on Initialized s,
p ) & (
J is
parahalting or
J is_halting_on IExec (
Ig,
p,
s),
p ) holds
(IExec ((Ig ";" J),p,s)) . f = (IExec (J,p,(IExec (Ig,p,s)))) . f
theorem
for
p being
Instruction-Sequence of
SCM+FSA for
s being
State of
SCM+FSA for
Ig being
good really-closed Program of
SCM+FSA for
J being
really-closed Program of
SCM+FSA st (
Ig is
parahalting or
Ig is_halting_on Initialized s,
p ) & (
J is
parahalting or
J is_halting_on IExec (
Ig,
p,
s),
p ) holds
DataPart (IExec ((Ig ";" J),p,s)) = DataPart (IExec (J,p,(IExec (Ig,p,s))))