definition
let x,
y be
object ;
coherence
{[x,y],[y,x]} is Function
commutativity
for b1 being Function
for x, y being object st b1 = {[x,y],[y,x]} holds
b1 = {[y,x],[x,y]}
;
end;
definition
let S be non
empty non
void ManySortedSign ;
let X be
V5()
ManySortedSet of the
carrier of
S;
let T be
X,
S -terms all_vars_including inheriting_operations free_in_itself MSAlgebra over
S;
attr T is
struct-invariant means
for
o being
OperSymbol of
S for
p being
Element of
Args (
o,
T) st
(Den (o,T)) . p = (Den (o,(Free (S,X)))) . p holds
for
s being
SortSymbol of
S for
x1,
x2 being
Element of
X . s holds
(Den (o,T)) . ((Hom (T,x1,x2)) # p) = (Den (o,(Free (S,X)))) . ((Hom (T,x1,x2)) # p);
end;
::
deftheorem defines
struct-invariant MSAFREE5:def 32 :
for S being non empty non void ManySortedSign
for X being V5() ManySortedSet of the carrier of S
for T being b2,b1 -terms all_vars_including inheriting_operations free_in_itself MSAlgebra over S holds
( T is struct-invariant iff for o being OperSymbol of S
for p being Element of Args (o,T) st (Den (o,T)) . p = (Den (o,(Free (S,X)))) . p holds
for s being SortSymbol of S
for x1, x2 being Element of X . s holds (Den (o,T)) . ((Hom (T,x1,x2)) # p) = (Den (o,(Free (S,X)))) . ((Hom (T,x1,x2)) # p) );
theorem Th112:
for
S being non
empty non
void ManySortedSign for
s being
SortSymbol of
S for
X being
V5()
ManySortedSet of the
carrier of
S for
x1,
x2 being
Element of
X . s for
R being
invariant stable terminating with_UN_property NF-var ManySortedRelation of
(Free (S,X)) holds
( ( for
t being
Element of
(NFAlgebra R) holds
((Hom ((Free (S,X)),x1,x2)) . (the_sort_of t)) . t = (Hom ((NFAlgebra R),x1,x2)) . t ) &
(Hom ((Free (S,X)),x1,x2)) || (NForms R) = Hom (
(NFAlgebra R),
x1,
x2) )
theorem Th113:
for
i being
Nat for
S being non
empty non
void ManySortedSign for
o being
OperSymbol of
S for
X being
V5()
ManySortedSet of the
carrier of
S for
t1,
t2 being
Element of
(Free (S,X)) for
p being
Element of
Args (
o,
(Free (S,X)))
for
R being
invariant stable terminating with_UN_property NF-var ManySortedRelation of
(Free (S,X)) st
i in dom p &
R . ((the_arity_of o) /. i) reduces t1,
t2 holds
R . (the_result_sort_of o) reduces (Den (o,(Free (S,X)))) . (p +* (i,t1)),
(Den (o,(Free (S,X)))) . (p +* (i,t2))
definition
let S be non
empty non
void ManySortedSign ;
let X be
V5()
ManySortedSet of the
carrier of
S;
let s be
SortSymbol of
S;
let x be
Element of
X . s;
let C be
context of
x;
existence
ex b1 being Function of ( the Sorts of (Free (S,X)) . s),( the Sorts of (Free (S,X)) . (the_sort_of C)) st
for t being Element of (Free (S,X)) st the_sort_of t = s holds
b1 . t = C -sub t
uniqueness
for b1, b2 being Function of ( the Sorts of (Free (S,X)) . s),( the Sorts of (Free (S,X)) . (the_sort_of C)) st ( for t being Element of (Free (S,X)) st the_sort_of t = s holds
b1 . t = C -sub t ) & ( for t being Element of (Free (S,X)) st the_sort_of t = s holds
b2 . t = C -sub t ) holds
b1 = b2
end;
theorem Th91:
for
m being
Element of
NAT for
S being non
empty non
void ManySortedSign for
o being
OperSymbol of
S for
Y being
infinite-yielding ManySortedSet of the
carrier of
S for
q being
Element of
Args (
o,
(Free (S,Y)))
for
s1,
s2 being
SortSymbol of
S for
V being
finite set st
m in dom q &
s1 = (the_arity_of o) /. m holds
ex
y being
Element of
Y . s1 ex
C being
context of
y ex
q1 being
Element of
Args (
o,
(Free (S,Y))) st
(
y nin V &
q1 = q +* (
m,
(y -term)) &
q1 is
y -context_including &
y -context_in q1 = y -term &
C = o -term q1 &
m = y -context_pos_in q1 &
transl C = transl (
o,
m,
q,
(Free (S,Y))) )
theorem
for
S being non
empty non
void ManySortedSign for
Y being
infinite-yielding ManySortedSet of the
carrier of
S for
v being
Element of
(Free (S,Y)) for
h being
Endomorphism of
Free (
S,
Y)
for
f being
vf-sequence of
v st
f <> {} holds
ex
B being non
empty FinSequence of the
carrier of
S ex
V1 being
b6 -sorts FinSequence of
Union Y st
(
dom B = dom f &
B = pr2 f &
V1 = pr1 f & ex
D being
b6 -sorts FinSequence of
(Free (S,Y)) ex
V2 being
b6 -sorts b7 -omitting b8 -omitting FinSequence of
Union Y st
( ( for
i being
Element of
dom B holds
D . i = h . ((V1 . i) -term) ) & ex
F being
b9 -context-sequence FinSequence of
(Free (S,Y)) st
(
F is
V1,
V2,
D -consequent-context-sequence &
(F . (In (1,(dom B)))) -sub ((V1 . (In (1,(dom B)))) -term) = v &
h . v = (F . (In ((len B),(dom B)))) -sub (D . (In ((len B),(dom B)))) ) ) )