definition
let K be
Ring;
let A be
Matrix of
K;
existence
ex b1 being Matrix of K st
( len b1 = len A & width b1 = width A & ( for i, j being Nat st [i,j] in Indices A holds
b1 * (i,j) = - (A * (i,j)) ) )
uniqueness
for b1, b2 being Matrix of K st len b1 = len A & width b1 = width A & ( for i, j being Nat st [i,j] in Indices A holds
b1 * (i,j) = - (A * (i,j)) ) & len b2 = len A & width b2 = width A & ( for i, j being Nat st [i,j] in Indices A holds
b2 * (i,j) = - (A * (i,j)) ) holds
b1 = b2
end;
definition
let K be
Ring;
let A,
B be
Matrix of
K;
existence
ex b1 being Matrix of K st
( len b1 = len A & width b1 = width A & ( for i, j being Nat st [i,j] in Indices A holds
b1 * (i,j) = (A * (i,j)) + (B * (i,j)) ) )
uniqueness
for b1, b2 being Matrix of K st len b1 = len A & width b1 = width A & ( for i, j being Nat st [i,j] in Indices A holds
b1 * (i,j) = (A * (i,j)) + (B * (i,j)) ) & len b2 = len A & width b2 = width A & ( for i, j being Nat st [i,j] in Indices A holds
b2 * (i,j) = (A * (i,j)) + (B * (i,j)) ) holds
b1 = b2
end;
theorem
for
n,
m being
Nat for
K being
Ring for
A being
Matrix of
n,
m,
K holds
A + (0. (K,n,m)) = A
theorem
for
n,
m being
Nat for
K being
Ring for
A being
Matrix of
n,
m,
K holds
A + (- A) = 0. (
K,
n,
m)
definition
let K be
Ring;
let A,
B be
Matrix of
K;
assume A1:
width A = len B
;
existence
ex b1 being Matrix of K st
( len b1 = len A & width b1 = width B & ( for i, j being Nat st [i,j] in Indices b1 holds
b1 * (i,j) = (Line (A,i)) "*" (Col (B,j)) ) )
uniqueness
for b1, b2 being Matrix of K st len b1 = len A & width b1 = width B & ( for i, j being Nat st [i,j] in Indices b1 holds
b1 * (i,j) = (Line (A,i)) "*" (Col (B,j)) ) & len b2 = len A & width b2 = width B & ( for i, j being Nat st [i,j] in Indices b2 holds
b2 * (i,j) = (Line (A,i)) "*" (Col (B,j)) ) holds
b1 = b2
end;
definition
let n,
k,
m be
Nat;
let K be
Ring;
let A be
Matrix of
n,
k,
K;
let B be
Matrix of
width A,
m,
K;
*redefine func A * B -> Matrix of
len A,
width B,
K;
coherence
A * B is Matrix of len A, width B,K
end;
definition
let K be
Ring;
let M be
Matrix of
K;
let a be
Element of
K;
existence
ex b1 being Matrix of K st
( len b1 = len M & width b1 = width M & ( for i, j being Nat st [i,j] in Indices M holds
b1 * (i,j) = a * (M * (i,j)) ) )
uniqueness
for b1, b2 being Matrix of K st len b1 = len M & width b1 = width M & ( for i, j being Nat st [i,j] in Indices M holds
b1 * (i,j) = a * (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) = a * (M * (i,j)) ) holds
b1 = b2
end;
Lm1:
for L being non empty right_complementable add-associative right_zeroed addLoopStr
for p being FinSequence of L st ( for i being Element of NAT st i in dom p holds
p . i = 0. L ) holds
Sum p = 0. L
theorem
for
K being
Field for
a1,
a2,
b1,
b2,
c1,
c2,
d1,
d2 being
Element of
K holds
((a1,b1) ][ (c1,d1)) * ((a2,b2) ][ (c2,d2)) = (
((a1 * a2) + (b1 * c2)),
((a1 * b2) + (b1 * d2)))
][ (
((c1 * a2) + (d1 * c2)),
((c1 * b2) + (d1 * d2)))
definition
let I,
J,
D be non
empty set ;
let G be
BinOp of
D;
let f be
Function of
I,
D;
let g be
Function of
J,
D;
*redefine func G * (
f,
g)
-> Function of
[:I,J:],
D;
coherence
G * (f,g) is Function of [:I,J:],D
by FINSEQOP:79;
end;
theorem Th23:
for
I,
J,
D being non
empty set for
F,
G being
BinOp of
D for
f being
Function of
I,
D for
g being
Function of
J,
D for
X being
Element of
Fin I for
Y being
Element of
Fin J st
F is
commutative &
F is
associative & (
[:Y,X:] <> {} or
F is
having_a_unity ) &
G is
commutative holds
F $$ (
[:X,Y:],
(G * (f,g)))
= F $$ (
[:Y,X:],
(G * (g,f)))
theorem Th24:
for
D,
I,
J being non
empty set for
F,
G being
BinOp of
D for
f being
Function of
I,
D for
g being
Function of
J,
D st
F is
commutative &
F is
associative holds
for
x being
Element of
I for
y being
Element of
J holds
F $$ (
[:{.x.},{.y.}:],
(G * (f,g)))
= F $$ (
{.x.},
(G [:] (f,(F $$ ({.y.},g)))))
theorem Th25:
for
D,
I,
J being non
empty set for
F,
G being
BinOp of
D for
f being
Function of
I,
D for
g being
Function of
J,
D for
X being
Element of
Fin I for
Y being
Element of
Fin J st
F is
commutative &
F is
associative &
F is
having_a_unity &
F is
having_an_inverseOp &
G is_distributive_wrt F holds
for
x being
Element of
I holds
F $$ (
[:{.x.},Y:],
(G * (f,g)))
= F $$ (
{.x.},
(G [:] (f,(F $$ (Y,g)))))
theorem Th26:
for
D,
I,
J being non
empty set for
F,
G being
BinOp of
D for
f being
Function of
I,
D for
g being
Function of
J,
D for
X being
Element of
Fin I for
Y being
Element of
Fin J st
F is
having_a_unity &
F is
commutative &
F is
associative &
F is
having_an_inverseOp &
G is_distributive_wrt F holds
F $$ (
[:X,Y:],
(G * (f,g)))
= F $$ (
X,
(G [:] (f,(F $$ (Y,g)))))
theorem
for
D,
I,
J being non
empty set for
F,
G being
BinOp of
D for
f being
Function of
I,
D for
g being
Function of
J,
D st
F is
commutative &
F is
associative &
G is
commutative holds
for
x being
Element of
I for
y being
Element of
J holds
F $$ (
[:{.x.},{.y.}:],
(G * (f,g)))
= F $$ (
{.y.},
(G [;] ((F $$ ({.x.},f)),g)))
theorem
for
D,
I,
J being non
empty set for
F,
G being
BinOp of
D for
f being
Function of
I,
D for
g being
Function of
J,
D for
X being
Element of
Fin I for
Y being
Element of
Fin J st
F is
having_a_unity &
F is
commutative &
F is
associative &
F is
having_an_inverseOp &
G is_distributive_wrt F &
G is
commutative holds
F $$ (
[:X,Y:],
(G * (f,g)))
= F $$ (
Y,
(G [;] ((F $$ (X,f)),g)))
definition
let n be
Nat;
let K be
Ring;
let M be
Matrix of
n,
K;
existence
ex b1 being Function of (Permutations n), the carrier of K st
for p being Element of Permutations n holds b1 . p = - (( the multF of K $$ (Path_matrix (p,M))),p)
uniqueness
for b1, b2 being Function of (Permutations n), the carrier of K st ( for p being Element of Permutations n holds b1 . p = - (( the multF of K $$ (Path_matrix (p,M))),p) ) & ( for p being Element of Permutations n holds b2 . p = - (( the multF of K $$ (Path_matrix (p,M))),p) ) holds
b1 = b2
end;