Lm01:
for a, b, c, d being Real st a <= b + c & b <= d holds
a <= d + c
Lm02:
for a, b, c, d being Real st a < b + c & b - c < d holds
a - d < 2 * c
theorem Th06:
for
a,
b being
Real st
a <> 0 holds
a * (b / (2 * a)) = b / 2
definition
let X be non
empty set ;
let f,
g be
Function of
X,
REAL;
existence
ex b1 being Function of X,REAL st
for x being Element of X holds b1 . x = min ((f . x),(g . x))
uniqueness
for b1, b2 being Function of X,REAL st ( for x being Element of X holds b1 . x = min ((f . x),(g . x)) ) & ( for x being Element of X holds b2 . x = min ((f . x),(g . x)) ) holds
b1 = b2
commutativity
for b1, f, g being Function of X,REAL st ( for x being Element of X holds b1 . x = min ((f . x),(g . x)) ) holds
for x being Element of X holds b1 . x = min ((g . x),(f . x))
;
existence
ex b1 being Function of X,REAL st
for x being Element of X holds b1 . x = max ((f . x),(g . x))
uniqueness
for b1, b2 being Function of X,REAL st ( for x being Element of X holds b1 . x = max ((f . x),(g . x)) ) & ( for x being Element of X holds b2 . x = max ((f . x),(g . x)) ) holds
b1 = b2
commutativity
for b1, f, g being Function of X,REAL st ( for x being Element of X holds b1 . x = max ((f . x),(g . x)) ) holds
for x being Element of X holds b1 . x = max ((g . x),(f . x))
;
end;
Lm03:
for X being non empty set st ex s being object st
for r being object st r in X holds
s = r holds
ex r being object st X = {r}
Lm04:
for I being non empty closed_interval Subset of REAL
for TD being tagged_division of I
for f being Function of I,REAL st f = chi (I,I) holds
tagged_sum (f,TD) = vol I