begin
Lm1:
for X, Y being finite set st X c= Y & card X = card Y holds
X = Y
Lm2:
for X, Y being finite set
for F being Function of X,Y st card X = card Y holds
( F is onto iff F is one-to-one )
theorem Th1:
begin
theorem Th2:
theorem Th3:
theorem Th4:
theorem
canceled;
theorem
canceled;
theorem
canceled;
:: deftheorem Def1 defines Rev AFINSQ_2:def 1 :
for p, b2 being XFinSequence holds
( b2 = Rev p iff ( len b2 = len p & ( for i being Nat st i in dom b2 holds
b2 . i = p . ((len p) - (i + 1)) ) ) );
theorem Th8:
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
:: deftheorem Def2 defines /^ AFINSQ_2:def 2 :
for p being XFinSequence
for n being Nat
for b3 being XFinSequence holds
( b3 = p /^ n iff ( len b3 = (len p) -' n & ( for m being Nat st m in dom b3 holds
b3 . m = p . (m + n) ) ) );
theorem Th15:
theorem Th16:
theorem Th17:
theorem Th18:
theorem Th19:
theorem Th20:
theorem Th21:
theorem
:: deftheorem defines mid AFINSQ_2:def 3 :
for p being XFinSequence
for k1, k2 being Nat holds mid (p,k1,k2) = (p | k2) /^ (k1 -' 1);
theorem Th23:
theorem
theorem Th25:
theorem
theorem
theorem
definition
canceled;
end;
:: deftheorem AFINSQ_2:def 4 :
canceled;
theorem
canceled;
theorem
canceled;
begin
definition
let X be
finite natural-membered set ;
func Sgm0 X -> XFinSequence of
NAT means :
Def5:
(
rng it = X & ( for
l,
m,
k1,
k2 being
Nat st
l < m &
m < len it &
k1 = it . l &
k2 = it . m holds
k1 < k2 ) );
existence
ex b1 being XFinSequence of NAT st
( rng b1 = X & ( for l, m, k1, k2 being Nat st l < m & m < len b1 & k1 = b1 . l & k2 = b1 . m holds
k1 < k2 ) )
uniqueness
for b1, b2 being XFinSequence of NAT st rng b1 = X & ( for l, m, k1, k2 being Nat st l < m & m < len b1 & k1 = b1 . l & k2 = b1 . m holds
k1 < k2 ) & rng b2 = X & ( for l, m, k1, k2 being Nat st l < m & m < len b2 & k1 = b2 . l & k2 = b2 . m holds
k1 < k2 ) holds
b1 = b2
end;
:: deftheorem Def5 defines Sgm0 AFINSQ_2:def 5 :
for X being finite natural-membered set
for b2 being XFinSequence of NAT holds
( b2 = Sgm0 X iff ( rng b2 = X & ( for l, m, k1, k2 being Nat st l < m & m < len b2 & k1 = b2 . l & k2 = b2 . m holds
k1 < k2 ) ) );
theorem Th31:
theorem Th32:
theorem Th33:
definition
let B1,
B2 be
set ;
pred B1 <N< B2 means :
Def6:
for
n,
m being
Nat st
n in B1 &
m in B2 holds
n < m;
end;
:: deftheorem Def6 defines <N< AFINSQ_2:def 6 :
for B1, B2 being set holds
( B1 <N< B2 iff for n, m being Nat st n in B1 & m in B2 holds
n < m );
definition
let B1,
B2 be
set ;
pred B1 <N= B2 means :
Def7:
for
n,
m being
Nat st
n in B1 &
m in B2 holds
n <= m;
end;
:: deftheorem Def7 defines <N= AFINSQ_2:def 7 :
for B1, B2 being set holds
( B1 <N= B2 iff for n, m being Nat st n in B1 & m in B2 holds
n <= m );
theorem Th34:
theorem
theorem Th36:
theorem
theorem Th38:
theorem
theorem Th40:
theorem Th41:
theorem Th42:
theorem Th43:
theorem Th44:
theorem Th45:
theorem Th46:
:: deftheorem defines SubXFinS AFINSQ_2:def 8 :
for f being XFinSequence
for B being set holds SubXFinS (f,B) = f * (Sgm0 (B /\ (len f)));
theorem Th47:
theorem
canceled;
:: deftheorem Def9 defines "**" AFINSQ_2:def 9 :
for D being non empty set
for F being XFinSequence st F is D -valued holds
for b being BinOp of D st ( b is having_a_unity or len F >= 1 ) holds
for b4 being Element of D holds
( ( b is having_a_unity & len F = 0 implies ( b4 = b "**" F iff b4 = the_unity_wrt b ) ) & ( ( not b is having_a_unity or not len F = 0 ) implies ( b4 = b "**" F iff ex f being Function of NAT,D st
( f . 0 = F . 0 & ( for n being Nat st n + 1 < len F holds
f . (n + 1) = b . ((f . n),(F . (n + 1))) ) & b4 = f . ((len F) - 1) ) ) ) );
theorem Th49:
theorem Th50:
theorem Th51:
theorem Th52:
theorem Th53:
theorem Th54:
theorem Th55:
theorem Th56:
theorem Th57:
theorem
theorem Th59:
Lm3:
for cF being complex-valued XFinSequence holds cF is COMPLEX -valued
Lm4:
for rF being real-valued XFinSequence holds rF is REAL -valued
:: deftheorem defines Sum AFINSQ_2:def 10 :
for F being XFinSequence holds Sum F = addcomplex "**" F;
theorem Th60:
theorem Th61:
theorem Th62:
theorem Th63:
theorem
theorem
theorem
theorem Th67:
theorem
theorem Th69:
theorem Th70:
theorem
theorem
theorem Th73:
theorem Th74:
theorem Th75:
theorem
theorem Th77:
theorem Th78:
theorem Th79:
theorem
theorem
theorem Th82:
theorem
theorem Th84:
:: deftheorem Def11 defines FlattenSeq AFINSQ_2:def 11 :
for D being set
for F being XFinSequence of D ^omega
for b3 being Element of D ^omega holds
( b3 = FlattenSeq F iff ex g being BinOp of (D ^omega) st
( ( for p, q being Element of D ^omega holds g . (p,q) = p ^ q ) & b3 = g "**" F ) );
theorem
theorem
theorem Th87:
theorem
theorem
theorem Th90:
theorem Th91:
theorem Th92:
theorem
theorem