Lm1:
2 |^ 0 = 1
by NEWTON:4;
Lm2:
2 |^ 2 = 2 * 2
by NEWTON:81;
Lm3:
2 |^ 3 = (2 * 2) * 2
by POLYEQ_5:2;
Lm4:
2 |^ 4 = ((2 * 2) * 2) * 2
by POLYEQ_5:3;
Lm5:
2 |^ 5 = (((2 * 2) * 2) * 2) * 2
by NUMBER02:1;
Lm6:
2 |^ 8 = ((((((2 * 2) * 2) * 2) * 2) * 2) * 2) * 2
by NUMBER02:4;
Lm7: 2 |^ (8 + 8) =
(2 |^ 8) * (2 |^ 8)
by NEWTON:8
.=
65536
by Lm6
;
Lm8:
1 mod 3 = 1
by NAT_D:24;
Lm9:
2 mod 3 = 2
by NAT_D:24;
4 = 1 + (3 * 1)
;
then Lm10:
4 mod 3 = 1 mod 3
by NAT_D:61;
theorem Th1:
for
n being
Nat holds
( not
n < 3 or
n = 0 or
n = 1 or
n = 2 )
theorem
for
n being
Nat holds
( not
n < 4 or
n = 0 or
n = 1 or
n = 2 or
n = 3 )
theorem Th3:
for
n being
Nat holds
( not
n < 5 or
n = 0 or
n = 1 or
n = 2 or
n = 3 or
n = 4 )
Lm13:
for n being positive Nat holds 3 divides (2 * (2 |^ (2 |^ n))) + 1
deffunc H1( Nat, Nat) -> set = ($1 * (2 |^ (2 |^ $2))) + 1;
theorem Th43:
for
m,
n being
Nat st (
m is
odd or
m = (2 * n) + 1 ) holds
(2 |^ m) mod 3
= 2
Lm18:
for n, x, y, z being positive Nat st x <= y & (n |^ x) + (n |^ y) = n |^ z holds
( n = 2 & y = x & z = x + 1 )
theorem Th49:
for
n,
x,
y,
z,
t being
positive Nat st
x <= y &
y <= z holds
(
((n |^ x) + (n |^ y)) + (n |^ z) = n |^ t iff ( (
n = 2 &
y = x &
z = x + 1 &
t = x + 2 ) or (
n = 3 &
y = x &
z = x &
t = x + 1 ) ) )
theorem Th50:
for
n,
x,
y,
z,
t being
positive Nat holds
(
((n |^ x) + (n |^ y)) + (n |^ z) = n |^ t iff ( (
n = 2 &
y = x &
z = x + 1 &
t = x + 2 ) or (
n = 2 &
y = x + 1 &
z = x &
t = x + 2 ) or (
n = 2 &
z = y &
x = y + 1 &
t = y + 2 ) or (
n = 3 &
y = x &
z = x &
t = x + 1 ) ) )
Lm19:
for x, y, z, t being positive Nat st (x ^2) + (5 * (y ^2)) = z ^2 & (5 * (x ^2)) + (y ^2) = t ^2 holds
ex x1, y1, z1, t1 being Nat st
( (x1 ^2) + (5 * (y1 ^2)) = z1 ^2 & (5 * (x1 ^2)) + (y1 ^2) = t1 ^2 & x1,y1 are_coprime )
Lm20:
for x, y, z, t being Nat holds
( not x,y are_coprime or (x ^2) + (5 * (y ^2)) <> z ^2 or (5 * (x ^2)) + (y ^2) <> t ^2 )
Lm21:
for x, y, z, t being positive Nat holds
( (x ^2) + (5 * (y ^2)) <> z ^2 or (5 * (x ^2)) + (y ^2) <> t ^2 )
Lm22:
for x, y, z, t being positive Nat st (x ^2) + (6 * (y ^2)) = z ^2 & (6 * (x ^2)) + (y ^2) = t ^2 holds
ex x1, y1, z1, t1 being Nat st
( (x1 ^2) + (6 * (y1 ^2)) = z1 ^2 & (6 * (x1 ^2)) + (y1 ^2) = t1 ^2 & x1,y1 are_coprime )
Lm23:
for x, y, z, t being Nat holds
( not x,y are_coprime or (x ^2) + (6 * (y ^2)) <> z ^2 or (6 * (x ^2)) + (y ^2) <> t ^2 )
Lm24:
for x, y, z, t being positive Nat holds
( (x ^2) + (6 * (y ^2)) <> z ^2 or (6 * (x ^2)) + (y ^2) <> t ^2 )