begin
:: deftheorem BILINEAR:def 1 :
canceled;
:: deftheorem defines NulForm BILINEAR:def 2 :
for K being non empty ZeroStr
for V, W being VectSpStr of K holds NulForm (V,W) = [: the carrier of V, the carrier of W:] --> (0. K);
definition
let K be non
empty addLoopStr ;
let V,
W be non
empty VectSpStr of
K;
let f,
g be
Form of
V,
W;
func f + g -> Form of
V,
W means :
Def3:
for
v being
Vector of
V for
w being
Vector of
W holds
it . (
v,
w)
= (f . (v,w)) + (g . (v,w));
existence
ex b1 being Form 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 Form 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;
:: deftheorem Def3 defines + BILINEAR:def 3 :
for K being non empty addLoopStr
for V, W being non empty VectSpStr of K
for f, g, b6 being Form of V,W holds
( b6 = f + g iff for v being Vector of V
for w being Vector of W holds b6 . (v,w) = (f . (v,w)) + (g . (v,w)) );
definition
let K be non
empty multMagma ;
let V,
W be non
empty VectSpStr of
K;
let f be
Form of
V,
W;
let a be
Element of
K;
func a * f -> Form of
V,
W means :
Def4:
for
v being
Vector of
V for
w being
Vector of
W holds
it . (
v,
w)
= a * (f . (v,w));
existence
ex b1 being Form 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 Form 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;
:: deftheorem Def4 defines * BILINEAR:def 4 :
for K being non empty multMagma
for V, W being non empty VectSpStr of K
for f being Form of V,W
for a being Element of K
for b6 being Form of V,W holds
( b6 = a * f iff for v being Vector of V
for w being Vector of W holds b6 . (v,w) = a * (f . (v,w)) );
definition
let K be non
empty addLoopStr ;
let V,
W be non
empty VectSpStr of
K;
let f be
Form of
V,
W;
func - f -> Form of
V,
W means :
Def5:
for
v being
Vector of
V for
w being
Vector of
W holds
it . (
v,
w)
= - (f . (v,w));
existence
ex b1 being Form 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 Form 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;
:: deftheorem Def5 defines - BILINEAR:def 5 :
for K being non empty addLoopStr
for V, W being non empty VectSpStr of K
for f, b5 being Form of V,W holds
( b5 = - f iff for v being Vector of V
for w being Vector of W holds b5 . (v,w) = - (f . (v,w)) );
:: deftheorem defines - BILINEAR:def 6 :
for K being non empty right_complementable add-associative right_zeroed left-distributive left_unital doubleLoopStr
for V, W being non empty VectSpStr of K
for f being Form of V,W holds - f = (- (1. K)) * f;
:: deftheorem defines - BILINEAR:def 7 :
for K being non empty addLoopStr
for V, W being non empty VectSpStr of K
for f, g being Form of V,W holds f - g = f + (- g);
definition
let K be non
empty addLoopStr ;
let V,
W be non
empty VectSpStr of
K;
let f,
g be
Form of
V,
W;
redefine func f - g means :
Def8:
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 Form 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;
:: deftheorem Def8 defines - BILINEAR:def 8 :
for K being non empty addLoopStr
for V, W being non empty VectSpStr of K
for f, g, b6 being Form of V,W holds
( b6 = f - g iff for v being Vector of V
for w being Vector of W holds b6 . (v,w) = (f . (v,w)) - (g . (v,w)) );
theorem
canceled;
theorem
theorem
theorem
theorem
theorem
theorem
theorem
Lm1:
now
let K be non
empty 1-sorted ;
for V, W being non empty VectSpStr of K
for f being Form of V,W
for v being Element of the carrier of V
for y being Element of W holds
( (curry f) . v is Functional of W & (curry' f) . y is Functional of V )let V,
W be non
empty VectSpStr of
K;
for f being Form of V,W
for v being Element of the carrier of V
for y being Element of W holds
( (curry f) . v is Functional of W & (curry' f) . y is Functional of V )let f be
Form of
V,
W;
for v being Element of the carrier of V
for y being Element of W holds
( (curry f) . v is Functional of W & (curry' f) . y is Functional of V )let v be
Element of the
carrier of
V;
for y being Element of W holds
( (curry f) . v is Functional of W & (curry' f) . y is Functional of V )let y be
Element of
W;
( (curry f) . v is Functional of W & (curry' f) . y is Functional of V )A1:
dom f = [: the carrier of V, the carrier of W:]
by FUNCT_2:def 1;
then consider g being
Function such that A2:
(curry f) . v = g
and A3:
(
dom g = the
carrier of
W &
rng g c= rng f )
and
for
y being
set st
y in the
carrier of
W holds
g . y = f . (
v,
y)
by FUNCT_5:36;
reconsider g =
g as
Function of the
carrier of
W, the
carrier of
K by A3, FUNCT_2:4, XBOOLE_1:1;
g = (curry f) . v
by A2;
hence
(curry f) . v is
Functional of
W
;
(curry' f) . y is Functional of Vconsider h being
Function such that A4:
(curry' f) . y = h
and A5:
(
dom h = the
carrier of
V &
rng h c= rng f )
and
for
x being
set st
x in the
carrier of
V holds
h . x = f . (
x,
y)
by A1, FUNCT_5:39;
reconsider h =
h as
Function of the
carrier of
V, the
carrier of
K by A5, FUNCT_2:4, XBOOLE_1:1;
h = (curry' f) . y
by A4;
hence
(curry' f) . y is
Functional of
V
;
verum
end;
begin
:: deftheorem defines FunctionalFAF BILINEAR:def 9 :
for K being non empty 1-sorted
for V, W being non empty VectSpStr of K
for f being Form of V,W
for v being Vector of V holds FunctionalFAF (f,v) = (curry f) . v;
:: deftheorem defines FunctionalSAF BILINEAR:def 10 :
for K being non empty 1-sorted
for V, W being non empty VectSpStr of K
for f being Form of V,W
for w being Vector of W holds FunctionalSAF (f,w) = (curry' f) . w;
theorem Th9:
theorem Th10:
theorem Th11:
theorem Th12:
theorem Th13:
theorem Th14:
theorem Th15:
theorem Th16:
theorem Th17:
theorem Th18:
theorem
theorem
begin
definition
let K be non
empty multMagma ;
let V,
W be non
empty VectSpStr of
K;
let f be
Functional of
V;
let g be
Functional of
W;
func FormFunctional (
f,
g)
-> Form of
V,
W means :
Def11:
for
v being
Vector of
V for
w being
Vector of
W holds
it . (
v,
w)
= (f . v) * (g . w);
existence
ex b1 being Form of V,W st
for v being Vector of V
for w being Vector of W holds b1 . (v,w) = (f . v) * (g . w)
uniqueness
for b1, b2 being Form of V,W st ( for v being Vector of V
for w being Vector of W holds b1 . (v,w) = (f . v) * (g . w) ) & ( for v being Vector of V
for w being Vector of W holds b2 . (v,w) = (f . v) * (g . w) ) holds
b1 = b2
end;
:: deftheorem Def11 defines FormFunctional BILINEAR:def 11 :
for K being non empty multMagma
for V, W being non empty VectSpStr of K
for f being Functional of V
for g being Functional of W
for b6 being Form of V,W holds
( b6 = FormFunctional (f,g) iff for v being Vector of V
for w being Vector of W holds b6 . (v,w) = (f . v) * (g . w) );
theorem Th21:
theorem Th22:
theorem
theorem
theorem Th25:
theorem Th26:
begin
:: deftheorem Def12 defines additiveFAF BILINEAR:def 12 :
for K being non empty addLoopStr
for V, W being non empty VectSpStr of K
for f being Form of V,W holds
( f is additiveFAF iff for v being Vector of V holds FunctionalFAF (f,v) is additive );
:: deftheorem Def13 defines additiveSAF BILINEAR:def 13 :
for K being non empty addLoopStr
for V, W being non empty VectSpStr of K
for f being Form of V,W holds
( f is additiveSAF iff for w being Vector of W holds FunctionalSAF (f,w) is additive );
:: deftheorem Def14 defines homogeneousFAF BILINEAR:def 14 :
for K being non empty multMagma
for V, W being non empty VectSpStr of K
for f being Form of V,W holds
( f is homogeneousFAF iff for v being Vector of V holds FunctionalFAF (f,v) is homogeneous );
:: deftheorem Def15 defines homogeneousSAF BILINEAR:def 15 :
for K being non empty multMagma
for V, W being non empty VectSpStr of K
for f being Form of V,W holds
( f is homogeneousSAF iff for w being Vector of W holds FunctionalSAF (f,w) is homogeneous );
theorem Th27:
theorem Th28:
theorem Th29:
theorem Th30:
theorem Th31:
theorem Th32:
theorem Th33:
theorem Th34:
theorem Th35:
theorem Th36:
theorem Th37:
theorem Th38:
theorem
for
K being non
empty right_complementable add-associative right_zeroed associative well-unital distributive doubleLoopStr for
V,
W being non
empty right_complementable add-associative right_zeroed vector-distributive scalar-distributive scalar-associative scalar-unital VectSpStr of
K for
v,
u being
Vector of
V for
w,
t being
Vector of
W for
a,
b being
Element of
K for
f being
bilinear-Form 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
K being non
empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr for
V,
W being
VectSp of
K for
v,
u being
Vector of
V for
w,
t being
Vector of
W for
a,
b being
Element of
K for
f being
bilinear-Form 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 Th41:
begin
:: deftheorem defines leftker BILINEAR:def 16 :
for K being ZeroStr
for V, W being non empty VectSpStr of K
for f being Form of V,W holds leftker f = { v where v is Vector of V : for w being Vector of W holds f . (v,w) = 0. K } ;
:: deftheorem defines rightker BILINEAR:def 17 :
for K being ZeroStr
for V, W being non empty VectSpStr of K
for f being Form of V,W holds rightker f = { w where w is Vector of W : for v being Vector of V holds f . (v,w) = 0. K } ;
:: deftheorem defines diagker BILINEAR:def 18 :
for K being ZeroStr
for V being non empty VectSpStr of K
for f being Form of V,V holds diagker f = { v where v is Vector of V : f . (v,v) = 0. K } ;
theorem
theorem Th43:
theorem Th44:
:: deftheorem Def19 defines LKer BILINEAR:def 19 :
for K being non empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr
for V being VectSp of K
for W being non empty VectSpStr of K
for f being additiveSAF homogeneousSAF Form of V,W
for b5 being non empty strict Subspace of V holds
( b5 = LKer f iff the carrier of b5 = leftker f );
:: deftheorem Def20 defines RKer BILINEAR:def 20 :
for K being non empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr
for V being non empty VectSpStr of K
for W being VectSp of K
for f being additiveFAF homogeneousFAF Form of V,W
for b5 being non empty strict Subspace of W holds
( b5 = RKer f iff the carrier of b5 = rightker f );
definition
let K be non
empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr ;
let V be
VectSp of
K;
let W be non
empty VectSpStr of
K;
let f be
additiveSAF homogeneousSAF Form of
V,
W;
func LQForm f -> additiveSAF homogeneousSAF Form of
(VectQuot (V,(LKer f))),
W means :
Def21:
for
A being
Vector of
(VectQuot (V,(LKer f))) for
w being
Vector of
W for
v being
Vector of
V st
A = v + (LKer f) holds
it . (
A,
w)
= f . (
v,
w);
existence
ex b1 being additiveSAF homogeneousSAF Form of (VectQuot (V,(LKer f))),W st
for A being Vector of (VectQuot (V,(LKer f)))
for w being Vector of W
for v being Vector of V st A = v + (LKer f) holds
b1 . (A,w) = f . (v,w)
uniqueness
for b1, b2 being additiveSAF homogeneousSAF Form of (VectQuot (V,(LKer f))),W st ( for A being Vector of (VectQuot (V,(LKer f)))
for w being Vector of W
for v being Vector of V st A = v + (LKer f) holds
b1 . (A,w) = f . (v,w) ) & ( for A being Vector of (VectQuot (V,(LKer f)))
for w being Vector of W
for v being Vector of V st A = v + (LKer f) holds
b2 . (A,w) = f . (v,w) ) holds
b1 = b2
end;
:: deftheorem Def21 defines LQForm BILINEAR:def 21 :
for K being non empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr
for V being VectSp of K
for W being non empty VectSpStr of K
for f being additiveSAF homogeneousSAF Form of V,W
for b5 being additiveSAF homogeneousSAF Form of (VectQuot (V,(LKer f))),W holds
( b5 = LQForm f iff for A being Vector of (VectQuot (V,(LKer f)))
for w being Vector of W
for v being Vector of V st A = v + (LKer f) holds
b5 . (A,w) = f . (v,w) );
definition
let K be non
empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr ;
let V be non
empty VectSpStr of
K;
let W be
VectSp of
K;
let f be
additiveFAF homogeneousFAF Form of
V,
W;
func RQForm f -> additiveFAF homogeneousFAF Form of
V,
(VectQuot (W,(RKer f))) means :
Def22:
for
A being
Vector of
(VectQuot (W,(RKer f))) for
v being
Vector of
V for
w being
Vector of
W st
A = w + (RKer f) holds
it . (
v,
A)
= f . (
v,
w);
existence
ex b1 being additiveFAF homogeneousFAF Form of V,(VectQuot (W,(RKer f))) st
for A being Vector of (VectQuot (W,(RKer f)))
for v being Vector of V
for w being Vector of W st A = w + (RKer f) holds
b1 . (v,A) = f . (v,w)
uniqueness
for b1, b2 being additiveFAF homogeneousFAF Form of V,(VectQuot (W,(RKer f))) st ( for A being Vector of (VectQuot (W,(RKer f)))
for v being Vector of V
for w being Vector of W st A = w + (RKer f) holds
b1 . (v,A) = f . (v,w) ) & ( for A being Vector of (VectQuot (W,(RKer f)))
for v being Vector of V
for w being Vector of W st A = w + (RKer f) holds
b2 . (v,A) = f . (v,w) ) holds
b1 = b2
end;
:: deftheorem Def22 defines RQForm BILINEAR:def 22 :
for K being non empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr
for V being non empty VectSpStr of K
for W being VectSp of K
for f being additiveFAF homogeneousFAF Form of V,W
for b5 being additiveFAF homogeneousFAF Form of V,(VectQuot (W,(RKer f))) holds
( b5 = RQForm f iff for A being Vector of (VectQuot (W,(RKer f)))
for v being Vector of V
for w being Vector of W st A = w + (RKer f) holds
b5 . (v,A) = f . (v,w) );
definition
let K be non
empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr ;
let V,
W be
VectSp of
K;
let f be
bilinear-Form of
V,
W;
func QForm f -> bilinear-Form of
(VectQuot (V,(LKer f))),
(VectQuot (W,(RKer f))) means :
Def23:
for
A being
Vector of
(VectQuot (V,(LKer f))) for
B being
Vector of
(VectQuot (W,(RKer f))) for
v being
Vector of
V for
w being
Vector of
W st
A = v + (LKer f) &
B = w + (RKer f) holds
it . (
A,
B)
= f . (
v,
w);
existence
ex b1 being bilinear-Form of (VectQuot (V,(LKer f))),(VectQuot (W,(RKer f))) st
for A being Vector of (VectQuot (V,(LKer f)))
for B being Vector of (VectQuot (W,(RKer f)))
for v being Vector of V
for w being Vector of W st A = v + (LKer f) & B = w + (RKer f) holds
b1 . (A,B) = f . (v,w)
uniqueness
for b1, b2 being bilinear-Form of (VectQuot (V,(LKer f))),(VectQuot (W,(RKer f))) st ( for A being Vector of (VectQuot (V,(LKer f)))
for B being Vector of (VectQuot (W,(RKer f)))
for v being Vector of V
for w being Vector of W st A = v + (LKer f) & B = w + (RKer f) holds
b1 . (A,B) = f . (v,w) ) & ( for A being Vector of (VectQuot (V,(LKer f)))
for B being Vector of (VectQuot (W,(RKer f)))
for v being Vector of V
for w being Vector of W st A = v + (LKer f) & B = w + (RKer f) holds
b2 . (A,B) = f . (v,w) ) holds
b1 = b2
end;
:: deftheorem Def23 defines QForm BILINEAR:def 23 :
for K being non empty right_complementable Abelian add-associative right_zeroed associative well-unital distributive doubleLoopStr
for V, W being VectSp of K
for f being bilinear-Form of V,W
for b5 being bilinear-Form of (VectQuot (V,(LKer f))),(VectQuot (W,(RKer f))) holds
( b5 = QForm f iff for A being Vector of (VectQuot (V,(LKer f)))
for B being Vector of (VectQuot (W,(RKer f)))
for v being Vector of V
for w being Vector of W st A = v + (LKer f) & B = w + (RKer f) holds
b5 . (A,B) = f . (v,w) );
theorem Th45:
theorem Th46:
theorem Th47:
theorem Th48:
theorem Th49:
theorem Th50:
theorem Th51:
theorem Th52:
theorem Th53:
theorem Th54:
theorem Th55:
theorem Th56:
theorem
:: deftheorem Def24 defines degenerated-on-left BILINEAR:def 24 :
for K being ZeroStr
for V, W being non empty VectSpStr of K
for f being Form of V,W holds
( f is degenerated-on-left iff leftker f <> {(0. V)} );
:: deftheorem Def25 defines degenerated-on-right BILINEAR:def 25 :
for K being ZeroStr
for V, W being non empty VectSpStr of K
for f being Form of V,W holds
( f is degenerated-on-right iff rightker f <> {(0. W)} );
begin
:: deftheorem Def26 defines symmetric BILINEAR:def 26 :
for K being 1-sorted
for V being VectSpStr of K
for f being Form of V,V holds
( f is symmetric iff for v, w being Vector of V holds f . (v,w) = f . (w,v) );
:: deftheorem Def27 defines alternating BILINEAR:def 27 :
for K being ZeroStr
for V being VectSpStr of K
for f being Form of V,V holds
( f is alternating iff for v being Vector of V holds f . (v,v) = 0. K );
registration
let K be non
empty ZeroStr ;
let V be non
empty VectSpStr of
K;
cluster non
empty Relation-like [: the carrier of V, the carrier of V:] -defined the
carrier of
K -valued Function-like V17(
[: the carrier of V, the carrier of V:])
V18(
[: the carrier of V, the carrier of V:], the
carrier of
K)
symmetric Element of
bool [:[: the carrier of V, the carrier of V:], the carrier of K:];
existence
ex b1 being Form of V,V st b1 is symmetric
cluster non
empty Relation-like [: the carrier of V, the carrier of V:] -defined the
carrier of
K -valued Function-like V17(
[: the carrier of V, the carrier of V:])
V18(
[: the carrier of V, the carrier of V:], the
carrier of
K)
alternating Element of
bool [:[: the carrier of V, the carrier of V:], the carrier of K:];
existence
ex b1 being Form of V,V st b1 is alternating
end;
registration
let K be non
empty right_complementable add-associative right_zeroed right-distributive doubleLoopStr ;
let V be non
empty VectSpStr of
K;
cluster non
empty Relation-like [: the carrier of V, the carrier of V:] -defined the
carrier of
K -valued Function-like V17(
[: the carrier of V, the carrier of V:])
V18(
[: the carrier of V, the carrier of V:], the
carrier of
K)
additiveFAF additiveSAF homogeneousFAF homogeneousSAF symmetric Element of
bool [:[: the carrier of V, the carrier of V:], the carrier of K:];
existence
ex b1 being Form of V,V st
( b1 is symmetric & b1 is additiveFAF & b1 is homogeneousFAF & b1 is additiveSAF & b1 is homogeneousSAF )
cluster non
empty Relation-like [: the carrier of V, the carrier of V:] -defined the
carrier of
K -valued Function-like V17(
[: the carrier of V, the carrier of V:])
V18(
[: the carrier of V, the carrier of V:], the
carrier of
K)
additiveFAF additiveSAF homogeneousFAF homogeneousSAF alternating Element of
bool [:[: the carrier of V, the carrier of V:], the carrier of K:];
existence
ex b1 being Form of V,V st
( b1 is alternating & b1 is additiveFAF & b1 is homogeneousFAF & b1 is additiveSAF & b1 is homogeneousSAF )
end;
theorem
theorem Th59:
:: deftheorem defines alternating BILINEAR:def 28 :
for K being Fanoian Field
for V being non empty VectSpStr of K
for f being additiveFAF additiveSAF Form of V,V holds
( f is alternating iff for v, w being Vector of V holds f . (v,w) = - (f . (w,v)) );
theorem