theorem Th18:
for
R being non
degenerated comRing for
m being
Nat for
x,
y being
Element of
R for
D being
Derivation of
R holds
LBZ0 (
D,
m,
x,
y)
= (LBZ1 (D,m,x,y)) + (LBZ2 (D,m,x,y))
theorem Th19:
for
R being non
degenerated comRing for
n being
Nat for
x,
y being
Element of
R for
D being
Derivation of
R holds
Sum (LBZ0 (D,n,x,y)) = (Sum (LBZ1 (D,n,x,y))) + (Sum (LBZ2 (D,n,x,y)))
theorem Th20:
for
R being non
degenerated comRing for
n being
Nat for
x,
y being
Element of
R for
D being
Derivation of
R holds
D * (LBZ0 (D,n,x,y)) = (Del ((LBZ2 (D,(n + 1),x,y)),(n + 1))) + (Del ((LBZ1 (D,(n + 1),x,y)),1))
Lm1:
for R being non degenerated comRing
for x, y being Element of R
for D being Derivation of R
for n being Nat st 1 <= n holds
(LBZ1 (D,n,x,y)) /. 1 = ((D |^ n) . x) * (D . y)
Lm2:
for R being non degenerated comRing
for x, y being Element of R
for D being Derivation of R
for n being Nat st 1 <= n holds
(LBZ2 (D,n,x,y)) /. n = (D . x) * ((D |^ n) . y)
theorem Th21:
for
R being non
degenerated comRing for
n being
Nat for
x,
y being
Element of
R for
D being
Derivation of
R holds
Sum (D * (LBZ0 (D,n,x,y))) = ((- ((LBZ1 (D,(n + 1),x,y)) /. 1)) + (Sum (LBZ0 (D,(n + 1),x,y)))) - ((LBZ2 (D,(n + 1),x,y)) /. (n + 1))
Lm3:
for R being domRing
for a being Element of R holds a | R = <%a%>
Lm4:
for R being domRing
for p being non constant Polynomial of R holds LM p = ((p . (deg p)) * (anpoly ((1. R),((deg p) -' 1)))) *' (anpoly ((1. R),1))