Lm1:
number_e <> 1
by TAYLOR_1:11;
Lm2:
for x, y being Real st x ^2 < 1 & y < 1 holds
(x ^2) * y < 1
Lm3:
for x being Real st 1 <= x holds
(x ^2) - 1 >= 0
Lm4:
for x being Real st x ^2 < 1 holds
(x + 1) / (1 - x) > 0
theorem Th15:
for
x being
Real st
0 < x &
x < 1 holds
(1 + x) / (1 - x) > 0
Lm5:
for x being Real st 0 < x & x < 1 holds
0 < 1 - (x ^2)
Lm6:
for x being Real holds (x ^2) + 1 > 0
theorem Th32:
for
t being
Real st
- 1
< t &
t < 1 holds
0 < (t + 1) / (1 - t)
Lm7:
for t being Real st ( 1 < t or t < - 1 ) holds
0 < (t + 1) / (t - 1)
Lm8:
for x being Real holds sqrt ((x ^2) + 1) > x
Lm9:
for x, y being Real holds ((sqrt ((x ^2) + 1)) * (sqrt ((y ^2) + 1))) - (x * y) > 0
Lm10:
for y being Real st 1 <= y holds
y + (sqrt ((y ^2) - 1)) > 0
Lm11:
for t being Real st 0 < t holds
- 1 < ((t ^2) - 1) / ((t ^2) + 1)
Lm12:
for t being Real st 0 < t & t <> 1 & not 1 < ((t ^2) + 1) / ((t ^2) - 1) holds
((t ^2) + 1) / ((t ^2) - 1) < - 1
Lm13:
for t being Real st 0 < t holds
0 < (2 * t) / (1 + (t ^2))
;
Lm14:
for t being Real st 0 < t holds
(2 * t) / (1 + (t ^2)) <= 1
Lm15:
for t being Real st 0 < t holds
(1 - (sqrt (1 + (t ^2)))) / t < 0
Lm16:
for t being Real st 0 < t & t <= 1 holds
0 <= 1 - (t ^2)
Lm17:
for t being Real st 0 < t & t <= 1 holds
0 <= 4 - (4 * (t ^2))
Lm18:
for t being Real st 0 < t & t <= 1 holds
0 < 1 + (sqrt (1 - (t ^2)))
Lm19:
for t being Real st 0 < t & t <= 1 holds
0 < (1 + (sqrt (1 - (t ^2)))) / t
Lm20:
for t being Real st 0 < t & t <> 1 holds
(2 * t) / ((t ^2) - 1) <> 0
Lm21:
for t being Real st t < 0 holds
(1 + (sqrt (1 + (t ^2)))) / t < 0