begin
definition
let M be
Matrix of
REAL;
attr M is
Positive means :
Def1:
for
i,
j being
Nat st
[i,j] in Indices M holds
M * (
i,
j)
> 0 ;
attr M is
Negative means :
Def2:
for
i,
j being
Nat st
[i,j] in Indices M holds
M * (
i,
j)
< 0 ;
attr M is
Nonpositive means :
Def3:
for
i,
j being
Nat st
[i,j] in Indices M holds
M * (
i,
j)
<= 0 ;
attr M is
Nonnegative means :
Def4:
for
i,
j being
Nat st
[i,j] in Indices M holds
M * (
i,
j)
>= 0 ;
end;
:: deftheorem Def1 defines Positive MATRIX10:def 1 :
for M being Matrix of REAL holds
( M is Positive iff for i, j being Nat st [i,j] in Indices M holds
M * (i,j) > 0 );
:: deftheorem Def2 defines Negative MATRIX10:def 2 :
for M being Matrix of REAL holds
( M is Negative iff for i, j being Nat st [i,j] in Indices M holds
M * (i,j) < 0 );
:: deftheorem Def3 defines Nonpositive MATRIX10:def 3 :
for M being Matrix of REAL holds
( M is Nonpositive iff for i, j being Nat st [i,j] in Indices M holds
M * (i,j) <= 0 );
:: deftheorem Def4 defines Nonnegative MATRIX10:def 4 :
for M being Matrix of REAL holds
( M is Nonnegative iff for i, j being Nat st [i,j] in Indices M holds
M * (i,j) >= 0 );
:: deftheorem Def5 defines is_less_than MATRIX10:def 5 :
for M1, M2 being Matrix of REAL holds
( M1 is_less_than M2 iff for i, j being Nat st [i,j] in Indices M1 holds
M1 * (i,j) < M2 * (i,j) );
:: deftheorem Def6 defines is_less_or_equal_with MATRIX10:def 6 :
for M1, M2 being Matrix of REAL holds
( M1 is_less_or_equal_with M2 iff for i, j being Nat st [i,j] in Indices M1 holds
M1 * (i,j) <= M2 * (i,j) );
definition
let M be
Matrix of
REAL;
func |:M:| -> Matrix of
REAL means :
Def7:
(
len it = len M &
width it = width M & ( for
i,
j being
Nat st
[i,j] in Indices M holds
it * (
i,
j)
= abs (M * (i,j)) ) );
existence
ex b1 being Matrix of REAL st
( len b1 = len M & width b1 = width M & ( for i, j being Nat st [i,j] in Indices M holds
b1 * (i,j) = abs (M * (i,j)) ) )
uniqueness
for b1, b2 being Matrix of REAL st len b1 = len M & width b1 = width M & ( for i, j being Nat st [i,j] in Indices M holds
b1 * (i,j) = abs (M * (i,j)) ) & len b2 = len M & width b2 = width M & ( for i, j being Nat st [i,j] in Indices M holds
b2 * (i,j) = abs (M * (i,j)) ) holds
b1 = b2
end;
:: deftheorem Def7 defines |: MATRIX10:def 7 :
for M, b2 being Matrix of REAL holds
( b2 = |:M:| iff ( len b2 = len M & width b2 = width M & ( for i, j being Nat st [i,j] in Indices M holds
b2 * (i,j) = abs (M * (i,j)) ) ) );
registration
let n be
Nat;
cluster (
n,
n)
--> 1
-> Positive Matrix of
n,
REAL ;
coherence
for b1 being Matrix of n, REAL st b1 = (n,n) --> 1 holds
b1 is Positive
cluster (
n,
n)
--> (- 1) -> Negative Matrix of
n,
REAL ;
coherence
for b1 being Matrix of n, REAL st b1 = (n,n) --> (- 1) holds
b1 is Negative
cluster (
n,
n)
--> (- 1) -> Nonpositive Matrix of
n,
REAL ;
coherence
for b1 being Matrix of n, REAL st b1 = (n,n) --> (- 1) holds
b1 is Nonpositive
cluster (
n,
n)
--> 1
-> Nonnegative Matrix of
n,
REAL ;
coherence
for b1 being Matrix of n, REAL st b1 = (n,n) --> 1 holds
b1 is Nonnegative
end;
Lm1:
for n being Nat
for M1, M2 being Matrix of n, REAL holds
( len M1 = len M2 & width M1 = width M2 )
theorem
theorem Th2:
theorem Th3:
theorem Th4:
theorem Th5:
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th36:
theorem
theorem
theorem
theorem
theorem
theorem Th42:
theorem
begin
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem