begin
Lm1:
for a, A being set st A /\ {a} <> {} holds
a in A
begin
theorem
theorem Th2:
theorem
theorem
theorem Th5:
theorem
theorem Th7:
theorem Th8:
Lm2:
for R being non trivial good Ring
for a being Data-Location of R
for p being PartState of (SCM R) st a in dom p holds
a in dom (NPP p)
theorem Th9:
for
n being
Element of
NAT for
R being non
trivial good Ring for
a,
b being
Data-Location of
R for
s1,
s2 being
State of
(SCM R) for
P1,
P2 being the
Instructions of
(SCM b2) -valued ManySortedSet of
NAT st not
R is
trivial holds
for
p being non
NAT -defined autonomic FinPartState of st
NPP p c= s1 &
NPP p c= s2 &
ProgramPart p c= P1 &
ProgramPart p c= P2 &
CurInstr (
P1,
(Comput (P1,s1,n)))
= a := b &
a in dom p holds
(Comput (P1,s1,n)) . b = (Comput (P2,s2,n)) . b
theorem Th10:
for
n being
Element of
NAT for
R being non
trivial good Ring for
a,
b being
Data-Location of
R for
s1,
s2 being
State of
(SCM R) for
P1,
P2 being the
Instructions of
(SCM b2) -valued ManySortedSet of
NAT st not
R is
trivial holds
for
p being non
NAT -defined autonomic FinPartState of st
NPP p c= s1 &
NPP p c= s2 &
ProgramPart p c= P1 &
ProgramPart p c= P2 &
CurInstr (
P1,
(Comput (P1,s1,n)))
= AddTo (
a,
b) &
a in dom p holds
((Comput (P1,s1,n)) . a) + ((Comput (P1,s1,n)) . b) = ((Comput (P2,s2,n)) . a) + ((Comput (P2,s2,n)) . b)
theorem Th11:
for
n being
Element of
NAT for
R being non
trivial good Ring for
a,
b being
Data-Location of
R for
s1,
s2 being
State of
(SCM R) for
P1,
P2 being the
Instructions of
(SCM b2) -valued ManySortedSet of
NAT st not
R is
trivial holds
for
p being non
NAT -defined autonomic FinPartState of st
NPP p c= s1 &
NPP p c= s2 &
ProgramPart p c= P1 &
ProgramPart p c= P2 &
CurInstr (
P1,
(Comput (P1,s1,n)))
= SubFrom (
a,
b) &
a in dom p holds
((Comput (P1,s1,n)) . a) - ((Comput (P1,s1,n)) . b) = ((Comput (P2,s2,n)) . a) - ((Comput (P2,s2,n)) . b)
theorem Th12:
for
n being
Element of
NAT for
R being non
trivial good Ring for
a,
b being
Data-Location of
R for
s1,
s2 being
State of
(SCM R) for
P1,
P2 being the
Instructions of
(SCM b2) -valued ManySortedSet of
NAT st not
R is
trivial holds
for
p being non
NAT -defined autonomic FinPartState of st
NPP p c= s1 &
NPP p c= s2 &
ProgramPart p c= P1 &
ProgramPart p c= P2 &
CurInstr (
P1,
(Comput (P1,s1,n)))
= MultBy (
a,
b) &
a in dom p holds
((Comput (P1,s1,n)) . a) * ((Comput (P1,s1,n)) . b) = ((Comput (P2,s2,n)) . a) * ((Comput (P2,s2,n)) . b)
theorem Th13:
for
n being
Element of
NAT for
R being non
trivial good Ring for
a being
Data-Location of
R for
loc being
Element of
NAT for
s1,
s2 being
State of
(SCM R) for
P1,
P2 being the
Instructions of
(SCM b2) -valued ManySortedSet of
NAT st not
R is
trivial holds
for
p being non
NAT -defined autonomic FinPartState of st
NPP p c= s1 &
NPP p c= s2 &
ProgramPart p c= P1 &
ProgramPart p c= P2 &
CurInstr (
P1,
(Comput (P1,s1,n)))
= a =0_goto loc &
loc <> succ (IC (Comput (P1,s1,n))) holds
(
(Comput (P1,s1,n)) . a = 0. R iff
(Comput (P2,s2,n)) . a = 0. R )
begin
theorem Th14:
for
k being
Element of
NAT for
R being non
trivial good Ring for
s1,
s2 being
State of
(SCM R) for
p being
autonomic FinPartState of
(SCM R) st
IC in dom p &
NPP p c= s1 &
NPP (Relocated (p,k)) c= s2 holds
for
P1,
P2 being the
Instructions of
(SCM b2) -valued ManySortedSet of
NAT st
ProgramPart p c= P1 &
Reloc (
(ProgramPart p),
k)
c= P2 holds
for
i being
Element of
NAT holds
(
(IC (Comput (P1,s1,i))) + k = IC (Comput (P2,s2,i)) &
IncAddr (
(CurInstr (P1,(Comput (P1,s1,i)))),
k)
= CurInstr (
P2,
(Comput (P2,s2,i))) &
(Comput (P1,s1,i)) | (dom (DataPart p)) = (Comput (P2,s2,i)) | (dom (DataPart p)) &
DataPart (Comput (P1,(s1 +* (DataPart s2)),i)) = DataPart (Comput (P2,s2,i)) )