Lm1:
for j being Integer holds
( j >= 0 or j = - 1 or j < - 1 )
Lm2:
for j being Integer holds
( j >= 1 or j = 0 or j < 0 )
Lm3:
for L being non empty almost_left_invertible well-unital distributive associative commutative doubleLoopStr
for a being Element of L
for i being Integer st 0 > i holds
pow (a,i) = (pow (a,|.i.|)) "
Lm4:
for L being non empty non degenerated almost_left_invertible well-unital distributive associative commutative doubleLoopStr
for i being Integer
for x being Element of L st i <= 0 holds
pow (x,i) = (pow (x,|.i.|)) "
Lm5:
for L being non empty almost_left_invertible well-unital distributive associative commutative doubleLoopStr
for i being Element of NAT holds pow ((1. L),i) = 1. L
Lm6:
for L being non empty well-unital doubleLoopStr
for n being Element of NAT holds (1. L) |^ n = 1. L
Lm7:
for L being non empty almost_left_invertible well-unital distributive associative commutative doubleLoopStr
for m being Element of NAT
for x being Element of L st x <> 0. L holds
(x |^ m) * ((x ") |^ m) = 1. L
Lm8:
for L being non empty non degenerated right_complementable almost_left_invertible left-distributive well-unital add-associative right_zeroed associative commutative doubleLoopStr
for k being Element of NAT
for x being Element of L st x <> 0. L holds
(x ") |^ k = (x |^ k) "
Lm9:
for L being non empty non degenerated right_complementable almost_left_invertible well-unital distributive add-associative right_zeroed associative commutative doubleLoopStr
for x being Element of L st x <> 0. L holds
for n being Element of NAT holds pow ((x "),n) = (pow (x,n)) "
Lm10:
for L being non empty almost_left_invertible well-unital distributive associative commutative doubleLoopStr
for x being Element of L
for m being Element of NAT st x <> 0. L & x |^ m = 1. L holds
(x ") |^ m = 1. L
Lm11:
for L being non empty non degenerated almost_left_invertible well-unital distributive associative commutative doubleLoopStr
for x being Element of L
for i being Element of NAT st x <> 0. L & (x ") |^ i = 1. L holds
x |^ i = 1. L
definition
let L be non
empty almost_left_invertible well-unital distributive associative commutative doubleLoopStr ;
let m be
Nat;
let x be
Element of
L;
existence
ex b1 being Matrix of m,L st
for i, j being Nat st 1 <= i & i <= m & 1 <= j & j <= m holds
b1 * (i,j) = pow (x,((i - 1) * (j - 1)))
uniqueness
for b1, b2 being Matrix of m,L st ( for i, j being Nat st 1 <= i & i <= m & 1 <= j & j <= m holds
b1 * (i,j) = pow (x,((i - 1) * (j - 1))) ) & ( for i, j being Nat st 1 <= i & i <= m & 1 <= j & j <= m holds
b2 * (i,j) = pow (x,((i - 1) * (j - 1))) ) holds
b1 = b2
end;
theorem Th35:
for
L being
Field for
m,
n being
Nat st
m > 0 holds
for
M being
Matrix of
m,
n,
L holds
(1. (L,m)) * M = M
Lm12:
for L being Field
for m being Element of NAT st m > 0 holds
for p, q being Polynomial of L holds (emb ((2 * m),L)) * ((1. (L,(2 * m))) * (mConv ((p *' q),(2 * m)))) = (emb ((2 * m),L)) * (mConv ((p *' q),(2 * m)))