begin
definition
let X,
Y,
Z be
RealNormSpace;
let f be
Element of
BoundedLinearOperators (
X,
Y);
let g be
Element of
BoundedLinearOperators (
Y,
Z);
func g * f -> Element of
BoundedLinearOperators (
X,
Z)
equals
(modetrans (g,Y,Z)) * (modetrans (f,X,Y));
correctness
coherence
(modetrans (g,Y,Z)) * (modetrans (f,X,Y)) is Element of BoundedLinearOperators (X,Z);
end;
:: deftheorem defines * NDIFF_2:def 1 :
for X, Y, Z being RealNormSpace
for f being Element of BoundedLinearOperators (X,Y)
for g being Element of BoundedLinearOperators (Y,Z) holds g * f = (modetrans (g,Y,Z)) * (modetrans (f,X,Y));
definition
let X,
Y,
Z be
RealNormSpace;
let f be
Point of
(R_NormSpace_of_BoundedLinearOperators (X,Y));
let g be
Point of
(R_NormSpace_of_BoundedLinearOperators (Y,Z));
func g * f -> Point of
(R_NormSpace_of_BoundedLinearOperators (X,Z)) equals
(modetrans (g,Y,Z)) * (modetrans (f,X,Y));
correctness
coherence
(modetrans (g,Y,Z)) * (modetrans (f,X,Y)) is Point of (R_NormSpace_of_BoundedLinearOperators (X,Z));
end;
:: deftheorem defines * NDIFF_2:def 2 :
for X, Y, Z being RealNormSpace
for f being Point of (R_NormSpace_of_BoundedLinearOperators (X,Y))
for g being Point of (R_NormSpace_of_BoundedLinearOperators (Y,Z)) holds g * f = (modetrans (g,Y,Z)) * (modetrans (f,X,Y));
theorem Th1:
theorem
theorem Th3:
:: deftheorem Def3 defines is_Gateaux_differentiable_in NDIFF_2:def 3 :
for S, T being non trivial RealNormSpace
for f being PartFunc of S,T
for x0, z being Point of S holds
( f is_Gateaux_differentiable_in x0,z iff ex N being Neighbourhood of x0 st
( N c= dom f & ex dv being Point of T st
for e being Real st e > 0 holds
ex d being Real st
( d > 0 & ( for h being Real st abs h < d & h <> 0 & (h * z) + x0 in N holds
||.(((h ") * ((f /. ((h * z) + x0)) - (f /. x0))) - dv).|| < e ) ) ) );
theorem Th4:
:: deftheorem Def4 defines Gateaux_diff NDIFF_2:def 4 :
for S, T being non trivial RealNormSpace
for f being PartFunc of S,T
for x0, z being Point of S st f is_Gateaux_differentiable_in x0,z holds
for b6 being Point of T holds
( b6 = Gateaux_diff (f,x0,z) iff ex N being Neighbourhood of x0 st
( N c= dom f & ( for e being Real st e > 0 holds
ex d being Real st
( d > 0 & ( for h being Real st abs h < d & h <> 0 & (h * z) + x0 in N holds
||.(((h ") * ((f /. ((h * z) + x0)) - (f /. x0))) - b6).|| < e ) ) ) ) );
theorem
theorem
theorem Th7:
theorem
theorem Th9:
theorem
theorem Th11:
theorem Th12:
theorem