definition
let P be non
empty Poset;
let S be non
empty non
void ManySortedSign ;
mode OrderedAlgFam of
P,
S -> MSAlgebra-Family of the
carrier of
P,
S means :
Def1:
ex
F being
ManySortedFunction of the
InternalRel of
P st
for
i,
j,
k being
Element of
P st
i >= j &
j >= k holds
ex
f1 being
ManySortedFunction of
(it . i),
(it . j) ex
f2 being
ManySortedFunction of
(it . j),
(it . k) st
(
f1 = F . (
j,
i) &
f2 = F . (
k,
j) &
F . (
k,
i)
= f2 ** f1 &
f1 is_homomorphism it . i,
it . j );
existence
ex b1 being MSAlgebra-Family of the carrier of P,S ex F being ManySortedFunction of the InternalRel of P st
for i, j, k being Element of P st i >= j & j >= k holds
ex f1 being ManySortedFunction of (b1 . i),(b1 . j) ex f2 being ManySortedFunction of (b1 . j),(b1 . k) st
( f1 = F . (j,i) & f2 = F . (k,j) & F . (k,i) = f2 ** f1 & f1 is_homomorphism b1 . i,b1 . j )
end;
::
deftheorem Def1 defines
OrderedAlgFam MSALIMIT:def 1 :
for P being non empty Poset
for S being non empty non void ManySortedSign
for b3 being MSAlgebra-Family of the carrier of P,S holds
( b3 is OrderedAlgFam of P,S iff ex F being ManySortedFunction of the InternalRel of P st
for i, j, k being Element of P st i >= j & j >= k holds
ex f1 being ManySortedFunction of (b3 . i),(b3 . j) ex f2 being ManySortedFunction of (b3 . j),(b3 . k) st
( f1 = F . (j,i) & f2 = F . (k,j) & F . (k,i) = f2 ** f1 & f1 is_homomorphism b3 . i,b3 . j ) );
definition
let P be non
empty Poset;
let S be non
empty non
void ManySortedSign ;
let OAF be
OrderedAlgFam of
P,
S;
let B be
Binding of
OAF;
existence
ex b1 being Binding of OAF st
for i, j being Element of P st i >= j holds
b1 . (j,i) = IFEQ (j,i,(id the Sorts of (OAF . i)),((bind (B,i,j)) ** (id the Sorts of (OAF . i))))
uniqueness
for b1, b2 being Binding of OAF st ( for i, j being Element of P st i >= j holds
b1 . (j,i) = IFEQ (j,i,(id the Sorts of (OAF . i)),((bind (B,i,j)) ** (id the Sorts of (OAF . i)))) ) & ( for i, j being Element of P st i >= j holds
b2 . (j,i) = IFEQ (j,i,(id the Sorts of (OAF . i)),((bind (B,i,j)) ** (id the Sorts of (OAF . i)))) ) holds
b1 = b2
end;
definition
let P be non
empty Poset;
let S be non
empty non
void ManySortedSign ;
let OAF be
OrderedAlgFam of
P,
S;
let B be
Binding of
OAF;
existence
ex b1 being strict MSSubAlgebra of product OAF st
for s being SortSymbol of S
for f being Element of (SORTS OAF) . s holds
( f in the Sorts of b1 . s iff for i, j being Element of P st i >= j holds
((bind (B,i,j)) . s) . (f . i) = f . j )
uniqueness
for b1, b2 being strict MSSubAlgebra of product OAF st ( for s being SortSymbol of S
for f being Element of (SORTS OAF) . s holds
( f in the Sorts of b1 . s iff for i, j being Element of P st i >= j holds
((bind (B,i,j)) . s) . (f . i) = f . j ) ) & ( for s being SortSymbol of S
for f being Element of (SORTS OAF) . s holds
( f in the Sorts of b2 . s iff for i, j being Element of P st i >= j holds
((bind (B,i,j)) . s) . (f . i) = f . j ) ) holds
b1 = b2
end;
Lm1:
for S being empty void ManySortedSign holds id the carrier of S, id the carrier' of S form_morphism_between S,S
Lm2:
for S being non empty void ManySortedSign holds id the carrier of S, id the carrier' of S form_morphism_between S,S
definition
let S1,
S2 be
ManySortedSign ;
existence
ex b1 being set st
for x being set holds
( x in b1 iff ex f, g being Function st
( x = [f,g] & f,g form_morphism_between S1,S2 ) )
uniqueness
for b1, b2 being set st ( for x being set holds
( x in b1 iff ex f, g being Function st
( x = [f,g] & f,g form_morphism_between S1,S2 ) ) ) & ( for x being set holds
( x in b2 iff ex f, g being Function st
( x = [f,g] & f,g form_morphism_between S1,S2 ) ) ) holds
b1 = b2
end;