definition
let IT be non
empty LatticeStr over
INT.Ring ;
attr IT is
Z_Lattice-like means :
defZLattice:
( ( for
x being
Vector of
IT st ( for
y being
Vector of
IT holds
<;x,y;> = 0 ) holds
x = 0. IT ) & ( for
x,
y being
Vector of
IT holds
<;x,y;> = <;y,x;> ) & ( for
x,
y,
z being
Vector of
IT for
a being
Element of
INT.Ring holds
(
<;(x + y),z;> = <;x,z;> + <;y,z;> &
<;(a * x),y;> = a * <;x,y;> ) ) );
end;
::
deftheorem defZLattice defines
Z_Lattice-like ZMODLAT1:def 3 :
for IT being non empty LatticeStr over INT.Ring holds
( IT is Z_Lattice-like iff ( ( for x being Vector of IT st ( for y being Vector of IT holds <;x,y;> = 0 ) holds
x = 0. IT ) & ( for x, y being Vector of IT holds <;x,y;> = <;y,x;> ) & ( for x, y, z being Vector of IT
for a being Element of INT.Ring holds
( <;(x + y),z;> = <;x,z;> + <;y,z;> & <;(a * x),y;> = a * <;x,y;> ) ) ) );
ZMtoZL1:
for V being Z_Module
for sc being Function of [: the carrier of V, the carrier of V:], the carrier of F_Real holds
( GenLat (V,sc) is Abelian & GenLat (V,sc) is add-associative & GenLat (V,sc) is right_zeroed & GenLat (V,sc) is right_complementable & GenLat (V,sc) is scalar-distributive & GenLat (V,sc) is vector-distributive & GenLat (V,sc) is scalar-associative & GenLat (V,sc) is scalar-unital )
registration
let V be
Z_Module;
let sc be
Function of
[: the carrier of V, the carrier of V:], the
carrier of
F_Real;
correctness
coherence
( GenLat (V,sc) is Abelian & GenLat (V,sc) is add-associative & GenLat (V,sc) is right_zeroed & GenLat (V,sc) is right_complementable & GenLat (V,sc) is scalar-distributive & GenLat (V,sc) is vector-distributive & GenLat (V,sc) is scalar-associative & GenLat (V,sc) is scalar-unital );
by ZMtoZL1;
end;
ZMtoZL2:
for V being free Z_Module
for sc being Function of [: the carrier of V, the carrier of V:], the carrier of F_Real holds GenLat (V,sc) is free
theorem ThNonTrivialLat1:
definition
let V,
W be non
empty ModuleStr over
INT.Ring ;
let f,
g be
FrForm of
V,
W;
existence
ex b1 being FrForm of V,W st
for v being Vector of V
for w being Vector of W holds b1 . (v,w) = (f . (v,w)) + (g . (v,w))
uniqueness
for b1, b2 being FrForm of V,W st ( for v being Vector of V
for w being Vector of W holds b1 . (v,w) = (f . (v,w)) + (g . (v,w)) ) & ( for v being Vector of V
for w being Vector of W holds b2 . (v,w) = (f . (v,w)) + (g . (v,w)) ) holds
b1 = b2
end;
definition
let V,
W be non
empty ModuleStr over
INT.Ring ;
let f be
FrForm of
V,
W;
let a be
Element of
F_Real;
existence
ex b1 being FrForm of V,W st
for v being Vector of V
for w being Vector of W holds b1 . (v,w) = a * (f . (v,w))
uniqueness
for b1, b2 being FrForm of V,W st ( for v being Vector of V
for w being Vector of W holds b1 . (v,w) = a * (f . (v,w)) ) & ( for v being Vector of V
for w being Vector of W holds b2 . (v,w) = a * (f . (v,w)) ) holds
b1 = b2
end;
definition
let V,
W be non
empty ModuleStr over
INT.Ring ;
let f be
FrForm of
V,
W;
existence
ex b1 being FrForm of V,W st
for v being Vector of V
for w being Vector of W holds b1 . (v,w) = - (f . (v,w))
uniqueness
for b1, b2 being FrForm of V,W st ( for v being Vector of V
for w being Vector of W holds b1 . (v,w) = - (f . (v,w)) ) & ( for v being Vector of V
for w being Vector of W holds b2 . (v,w) = - (f . (v,w)) ) holds
b1 = b2
end;
definition
let V,
W be non
empty ModuleStr over
INT.Ring ;
let f,
g be
FrForm of
V,
W;
redefine func f - g means :
Def7:
for
v being
Vector of
V for
w being
Vector of
W holds
it . (
v,
w)
= (f . (v,w)) - (g . (v,w));
compatibility
for b1 being FrForm of V,W holds
( b1 = f - g iff for v being Vector of V
for w being Vector of W holds b1 . (v,w) = (f . (v,w)) - (g . (v,w)) )
end;
theorem
for
V,
W being non
empty right_complementable vector-distributive scalar-distributive scalar-associative scalar-unital add-associative right_zeroed ModuleStr over
INT.Ring for
v,
u being
Vector of
V for
w,
t being
Vector of
W for
a,
b being
Element of
INT.Ring for
f being
bilinear-FrForm of
V,
W holds
f . (
(v + (a * u)),
(w + (b * t)))
= ((f . (v,w)) + (b * (f . (v,t)))) + ((a * (f . (u,w))) + (a * (b * (f . (u,t)))))
theorem
for
V,
W being
Z_Module for
v,
u being
Vector of
V for
w,
t being
Vector of
W for
a,
b being
Element of
INT.Ring for
f being
bilinear-FrForm of
V,
W holds
f . (
(v - (a * u)),
(w - (b * t)))
= ((f . (v,w)) - (b * (f . (v,t)))) - ((a * (f . (u,w))) - (a * (b * (f . (u,t)))))
definition
let V1,
V2 be
free finite-rank Z_Module;
let b1 be
OrdBasis of
V1;
let b2 be
OrdBasis of
V2;
let f be
bilinear-FrForm of
V1,
V2;
existence
ex b1 being Matrix of len b1, len b2,F_Real st
for i, j being Nat st i in dom b1 & j in dom b2 holds
b1 * (i,j) = f . ((b1 /. i),(b2 /. j))
uniqueness
for b1, b2 being Matrix of len b1, len b2,F_Real st ( for i, j being Nat st i in dom b1 & j in dom b2 holds
b1 * (i,j) = f . ((b1 /. i),(b2 /. j)) ) & ( for i, j being Nat st i in dom b1 & j in dom b2 holds
b2 * (i,j) = f . ((b1 /. i),(b2 /. j)) ) holds
b1 = b2
end;
theorem MLT1:
for
m,
l,
n being
Nat for
S being
Matrix of
l,
m,
INT.Ring for
T being
Matrix of
m,
n,
INT.Ring for
S1 being
Matrix of
l,
m,
F_Real for
T1 being
Matrix of
m,
n,
F_Real st
S = S1 &
T = T1 &
0 < l &
0 < m holds
S * T = S1 * T1
theorem ThMBF3:
for
V being
free finite-rank Z_Module for
b1,
b2 being
OrdBasis of
V for
f being
bilinear-FrForm of
V,
V st
0 < rank V holds
BilinearM (
f,
b2,
b2)
= ((inttorealM (AutMt ((id V),b2,b1))) * (BilinearM (f,b1,b1))) * ((inttorealM (AutMt ((id V),b2,b1))) @)
ThIntLatZ:
for L being INTegral Z_Lattice holds GramDet L is Integer