MeanL:
for f being heterogeneous real-valued FinSequence holds MeanLess f <> {}
MeanM:
for f being heterogeneous real-valued FinSequence holds MeanMore f <> {}
registration
let f be
real-valued FinSequence;
let i,
j be
Nat;
let a,
b be
Real;
coherence
( Replace (f,i,j,a,b) is real-valued & Replace (f,i,j,a,b) is FinSequence-like )
;
end;
theorem ReplacePositive2:
definition
let f be
heterogeneous non
empty real-valued positive FinSequence;
existence
ex b1 being real-valued FinSequence ex i, j being Nat st
( i = the Element of MeanLess f & j = the Element of MeanMore f & b1 = Replace (f,i,j,(Mean f),(((f . i) + (f . j)) - (Mean f))) )
uniqueness
for b1, b2 being real-valued FinSequence st ex i, j being Nat st
( i = the Element of MeanLess f & j = the Element of MeanMore f & b1 = Replace (f,i,j,(Mean f),(((f . i) + (f . j)) - (Mean f))) ) & ex i, j being Nat st
( i = the Element of MeanLess f & j = the Element of MeanMore f & b2 = Replace (f,i,j,(Mean f),(((f . i) + (f . j)) - (Mean f))) ) holds
b1 = b2
;
end;