begin
theorem Th1:
theorem Th2:
begin
:: deftheorem defines SVF1 PDIFF_2:def 1 :
for n, i being Element of NAT
for f being PartFunc of (REAL n),REAL
for z being Element of REAL n holds SVF1 (i,f,z) = f * (reproj (i,z));
theorem Th3:
theorem Th4:
theorem Th5:
theorem Th6:
theorem
for
x0,
y0 being
Real for
z being
Element of
REAL 2
for
f being
PartFunc of
(REAL 2),
REAL st
z = <*x0,y0*> &
f is_partial_differentiable_in z,1 holds
ex
N being
Neighbourhood of
x0 st
(
N c= dom (SVF1 (1,f,z)) & ex
L being
LINEAR ex
R being
REST st
for
x being
Real st
x in N holds
((SVF1 (1,f,z)) . x) - ((SVF1 (1,f,z)) . x0) = (L . (x - x0)) + (R . (x - x0)) )
theorem
for
x0,
y0 being
Real for
z being
Element of
REAL 2
for
f being
PartFunc of
(REAL 2),
REAL st
z = <*x0,y0*> &
f is_partial_differentiable_in z,2 holds
ex
N being
Neighbourhood of
y0 st
(
N c= dom (SVF1 (2,f,z)) & ex
L being
LINEAR ex
R being
REST st
for
y being
Real st
y in N holds
((SVF1 (2,f,z)) . y) - ((SVF1 (2,f,z)) . y0) = (L . (y - y0)) + (R . (y - y0)) )
theorem Th9:
for
f being
PartFunc of
(REAL 2),
REAL for
z being
Element of
REAL 2 holds
(
f is_partial_differentiable_in z,1 iff ex
x0,
y0 being
Real st
(
z = <*x0,y0*> & ex
N being
Neighbourhood of
x0 st
(
N c= dom (SVF1 (1,f,z)) & ex
L being
LINEAR ex
R being
REST st
for
x being
Real st
x in N holds
((SVF1 (1,f,z)) . x) - ((SVF1 (1,f,z)) . x0) = (L . (x - x0)) + (R . (x - x0)) ) ) )
theorem Th10:
for
f being
PartFunc of
(REAL 2),
REAL for
z being
Element of
REAL 2 holds
(
f is_partial_differentiable_in z,2 iff ex
x0,
y0 being
Real st
(
z = <*x0,y0*> & ex
N being
Neighbourhood of
y0 st
(
N c= dom (SVF1 (2,f,z)) & ex
L being
LINEAR ex
R being
REST st
for
y being
Real st
y in N holds
((SVF1 (2,f,z)) . y) - ((SVF1 (2,f,z)) . y0) = (L . (y - y0)) + (R . (y - y0)) ) ) )
Lm1:
for x0, y0, r being Real
for z being Element of REAL 2
for f being PartFunc of (REAL 2),REAL st z = <*x0,y0*> & f is_partial_differentiable_in z,1 holds
( r = diff ((SVF1 (1,f,z)),x0) iff ex x0, y0 being Real st
( z = <*x0,y0*> & ex N being Neighbourhood of x0 st
( N c= dom (SVF1 (1,f,z)) & ex L being LINEAR ex R being REST st
( r = L . 1 & ( for x being Real st x in N holds
((SVF1 (1,f,z)) . x) - ((SVF1 (1,f,z)) . x0) = (L . (x - x0)) + (R . (x - x0)) ) ) ) ) )
Lm2:
for x0, y0, r being Real
for z being Element of REAL 2
for f being PartFunc of (REAL 2),REAL st z = <*x0,y0*> & f is_partial_differentiable_in z,2 holds
( r = diff ((SVF1 (2,f,z)),y0) iff ex x0, y0 being Real st
( z = <*x0,y0*> & ex N being Neighbourhood of y0 st
( N c= dom (SVF1 (2,f,z)) & ex L being LINEAR ex R being REST st
( r = L . 1 & ( for y being Real st y in N holds
((SVF1 (2,f,z)) . y) - ((SVF1 (2,f,z)) . y0) = (L . (y - y0)) + (R . (y - y0)) ) ) ) ) )
theorem Th11:
for
x0,
y0,
r being
Real for
z being
Element of
REAL 2
for
f being
PartFunc of
(REAL 2),
REAL st
z = <*x0,y0*> &
f is_partial_differentiable_in z,1 holds
(
r = partdiff (
f,
z,1) iff ex
x0,
y0 being
Real st
(
z = <*x0,y0*> & ex
N being
Neighbourhood of
x0 st
(
N c= dom (SVF1 (1,f,z)) & ex
L being
LINEAR ex
R being
REST st
(
r = L . 1 & ( for
x being
Real st
x in N holds
((SVF1 (1,f,z)) . x) - ((SVF1 (1,f,z)) . x0) = (L . (x - x0)) + (R . (x - x0)) ) ) ) ) )
theorem Th12:
for
x0,
y0,
r being
Real for
z being
Element of
REAL 2
for
f being
PartFunc of
(REAL 2),
REAL st
z = <*x0,y0*> &
f is_partial_differentiable_in z,2 holds
(
r = partdiff (
f,
z,2) iff ex
x0,
y0 being
Real st
(
z = <*x0,y0*> & ex
N being
Neighbourhood of
y0 st
(
N c= dom (SVF1 (2,f,z)) & ex
L being
LINEAR ex
R being
REST st
(
r = L . 1 & ( for
y being
Real st
y in N holds
((SVF1 (2,f,z)) . y) - ((SVF1 (2,f,z)) . y0) = (L . (y - y0)) + (R . (y - y0)) ) ) ) ) )
theorem
theorem
:: deftheorem Def2 defines is_partial_differentiable`1_on PDIFF_2:def 2 :
for f being PartFunc of (REAL 2),REAL
for Z being set holds
( f is_partial_differentiable`1_on Z iff ( Z c= dom f & ( for z being Element of REAL 2 st z in Z holds
f | Z is_partial_differentiable_in z,1 ) ) );
:: deftheorem Def3 defines is_partial_differentiable`2_on PDIFF_2:def 3 :
for f being PartFunc of (REAL 2),REAL
for Z being set holds
( f is_partial_differentiable`2_on Z iff ( Z c= dom f & ( for z being Element of REAL 2 st z in Z holds
f | Z is_partial_differentiable_in z,2 ) ) );
theorem
theorem
definition
let f be
PartFunc of
(REAL 2),
REAL;
let Z be
set ;
assume A1:
f is_partial_differentiable`1_on Z
;
func f `partial1| Z -> PartFunc of
(REAL 2),
REAL means
(
dom it = Z & ( for
z being
Element of
REAL 2 st
z in Z holds
it . z = partdiff (
f,
z,1) ) );
existence
ex b1 being PartFunc of (REAL 2),REAL st
( dom b1 = Z & ( for z being Element of REAL 2 st z in Z holds
b1 . z = partdiff (f,z,1) ) )
uniqueness
for b1, b2 being PartFunc of (REAL 2),REAL st dom b1 = Z & ( for z being Element of REAL 2 st z in Z holds
b1 . z = partdiff (f,z,1) ) & dom b2 = Z & ( for z being Element of REAL 2 st z in Z holds
b2 . z = partdiff (f,z,1) ) holds
b1 = b2
end;
:: deftheorem defines `partial1| PDIFF_2:def 4 :
for f being PartFunc of (REAL 2),REAL
for Z being set st f is_partial_differentiable`1_on Z holds
for b3 being PartFunc of (REAL 2),REAL holds
( b3 = f `partial1| Z iff ( dom b3 = Z & ( for z being Element of REAL 2 st z in Z holds
b3 . z = partdiff (f,z,1) ) ) );
definition
let f be
PartFunc of
(REAL 2),
REAL;
let Z be
set ;
assume A1:
f is_partial_differentiable`2_on Z
;
func f `partial2| Z -> PartFunc of
(REAL 2),
REAL means
(
dom it = Z & ( for
z being
Element of
REAL 2 st
z in Z holds
it . z = partdiff (
f,
z,2) ) );
existence
ex b1 being PartFunc of (REAL 2),REAL st
( dom b1 = Z & ( for z being Element of REAL 2 st z in Z holds
b1 . z = partdiff (f,z,2) ) )
uniqueness
for b1, b2 being PartFunc of (REAL 2),REAL st dom b1 = Z & ( for z being Element of REAL 2 st z in Z holds
b1 . z = partdiff (f,z,2) ) & dom b2 = Z & ( for z being Element of REAL 2 st z in Z holds
b2 . z = partdiff (f,z,2) ) holds
b1 = b2
end;
:: deftheorem defines `partial2| PDIFF_2:def 5 :
for f being PartFunc of (REAL 2),REAL
for Z being set st f is_partial_differentiable`2_on Z holds
for b3 being PartFunc of (REAL 2),REAL holds
( b3 = f `partial2| Z iff ( dom b3 = Z & ( for z being Element of REAL 2 st z in Z holds
b3 . z = partdiff (f,z,2) ) ) );
begin
theorem
for
f being
PartFunc of
(REAL 2),
REAL for
z0 being
Element of
REAL 2
for
N being
Neighbourhood of
(proj (1,2)) . z0 st
f is_partial_differentiable_in z0,1 &
N c= dom (SVF1 (1,f,z0)) holds
for
h being
convergent_to_0 Real_Sequence for
c being
V20()
Real_Sequence st
rng c = {((proj (1,2)) . z0)} &
rng (h + c) c= N holds
(
(h ") (#) (((SVF1 (1,f,z0)) /* (h + c)) - ((SVF1 (1,f,z0)) /* c)) is
convergent &
partdiff (
f,
z0,1)
= lim ((h ") (#) (((SVF1 (1,f,z0)) /* (h + c)) - ((SVF1 (1,f,z0)) /* c))) )
theorem
for
f being
PartFunc of
(REAL 2),
REAL for
z0 being
Element of
REAL 2
for
N being
Neighbourhood of
(proj (2,2)) . z0 st
f is_partial_differentiable_in z0,2 &
N c= dom (SVF1 (2,f,z0)) holds
for
h being
convergent_to_0 Real_Sequence for
c being
V20()
Real_Sequence st
rng c = {((proj (2,2)) . z0)} &
rng (h + c) c= N holds
(
(h ") (#) (((SVF1 (2,f,z0)) /* (h + c)) - ((SVF1 (2,f,z0)) /* c)) is
convergent &
partdiff (
f,
z0,2)
= lim ((h ") (#) (((SVF1 (2,f,z0)) /* (h + c)) - ((SVF1 (2,f,z0)) /* c))) )
theorem
theorem
theorem
theorem