theorem Th1:
for
r,
s being
Real st
0 <= r &
s * s < r * r holds
s < r
theorem Th2:
for
r,
s being
Real st 1
< r &
r * r <= s holds
r < s
theorem Th3:
for
a,
n being
Nat st
a > 1 holds
a |^ n > n
theorem Th9:
for
i,
j,
k,
l being
Nat st
i = (j * k) + l &
l < j &
0 < l holds
not
j divides i
Lm1:
for p being Nat holds
( ( p <= 1 or ex n being Element of NAT st
( n divides p & 1 < n & n * n <= p & n is prime ) ) iff not p is prime )
Lm2:
for n being Nat st n < 5 & n is prime & not n = 2 holds
n = 3
Lm3:
for k being Nat st k < 25 holds
for n being Nat st n * n <= k & n is prime & not n = 2 holds
n = 3
Lm4:
( not 6 is prime & not 8 is prime & not 9 is prime & not 10 is prime & not 12 is prime & not 14 is prime & not 15 is prime & not 16 is prime & not 18 is prime & not 20 is prime & not 21 is prime & not 22 is prime & not 24 is prime & not 25 is prime & not 26 is prime & not 27 is prime & not 28 is prime )
Lm5:
for n being Nat st n < 29 & n is prime & not n = 2 & not n = 3 & not n = 5 & not n = 7 & not n = 11 & not n = 13 & not n = 17 & not n = 19 holds
n = 23
Lm6:
for k being Nat st k < 841 holds
for n being Nat st n * n <= k & n is prime & not n = 2 & not n = 3 & not n = 5 & not n = 7 & not n = 11 & not n = 13 & not n = 17 & not n = 19 holds
n = 23
Lm7:
for n being Element of NAT st 1 <= n & n < 4001 holds
ex p being Prime st
( n < p & p <= 2 * n )
Lm8:
for n, r being Element of NAT
for p being Prime
for f being FinSequence of REAL st p |^ r <= 2 * n & 2 * n < p |^ (r + 1) & len f = 2 * n & ( for k being Element of NAT st k in dom f holds
f . k = [\((2 * n) / (p |^ k))/] - (2 * [\(n / (p |^ k))/]) ) holds
Sum f <= r
Lm9:
for n being Element of NAT
for p being Prime st n >= 3 holds
( ( p > 2 * n implies p |-count ((2 * n) choose n) = 0 ) & ( n < p & p <= 2 * n implies p |-count ((2 * n) choose n) <= 1 ) & ( (2 * n) / 3 < p & p <= n implies p |-count ((2 * n) choose n) = 0 ) & ( sqrt (2 * n) < p & p <= (2 * n) / 3 implies p |-count ((2 * n) choose n) <= 1 ) & ( p <= sqrt (2 * n) implies p |^ (p |-count ((2 * n) choose n)) <= 2 * n ) )
Lm10:
for n, m being Element of NAT st m = (2 * n) choose n & n >= 3 holds
m = ((Product (Sgm { (p |^ (p |-count m)) where p is prime Element of NAT : ( p <= sqrt (2 * n) & p |-count m > 0 ) } )) * (Product (Sgm { (p |^ (p |-count m)) where p is prime Element of NAT : ( sqrt (2 * n) < p & p <= (2 * n) / 3 & p |-count m > 0 ) } ))) * (Product (Sgm { (p |^ (p |-count m)) where p is prime Element of NAT : ( n < p & p <= 2 * n & p |-count m > 0 ) } ))
Lm11:
for n, m being Element of NAT st m = (2 * n) choose n & n >= 3 holds
Product (Sgm { (p |^ (p |-count m)) where p is prime Element of NAT : ( p <= sqrt (2 * n) & p |-count m > 0 ) } ) <= (2 * n) to_power (sqrt (2 * n))
theorem
for
k being
Nat st
k < 25 holds
for
n being
Nat st
n * n <= k &
n is
prime & not
n = 2 holds
n = 3
by Lm3;
theorem
for
n being
Nat st
n < 29 &
n is
prime & not
n = 2 & not
n = 3 & not
n = 5 & not
n = 7 & not
n = 11 & not
n = 13 & not
n = 17 & not
n = 19 holds
n = 23
by Lm5;
theorem
for
k being
Nat st
k < 841 holds
for
n being
Nat st
n * n <= k &
n is
prime & not
n = 2 & not
n = 3 & not
n = 5 & not
n = 7 & not
n = 11 & not
n = 13 & not
n = 17 & not
n = 19 holds
n = 23
by Lm6;