begin
theorem Th1:
for
p,
q being
Prime for
k being
Nat holds
( not
k divides p * q or
k = 1 or
k = p or
k = q or
k = p * q )
:: deftheorem Def1 defines Safe GR_CY_3:def 1 :
for p being Nat holds
( p is Safe iff ex sgp being Prime st (2 * sgp) + 1 = p );
theorem Th2:
theorem Th3:
theorem Th4:
theorem Th5:
theorem
theorem
theorem
:: deftheorem Def2 defines Sophie_Germain GR_CY_3:def 2 :
for p being Nat holds
( p is Sophie_Germain iff (2 * p) + 1 is Prime );
theorem
theorem Th10:
Lm1:
for p being Nat st p > 2 holds
(2 * p) + 1 > 5
theorem Th11:
theorem
theorem Th13:
theorem Th14:
theorem
:: deftheorem defines Mersenne GR_CY_3:def 3 :
for n being Nat holds Mersenne n = (2 |^ n) - 1;
Lm2:
2 |^ 2 = 4
Lm3:
2 |^ 3 = 8
Lm4:
2 |^ 4 = 16
Lm5:
2 |^ 8 = 256
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th27:
Lm6:
for a, p being Nat st p > 1 & (a |^ p) - 1 is Prime holds
a > 1
theorem Th28:
theorem
theorem Th30:
theorem Th31:
theorem
theorem
Lm7:
for n being Nat
for a being Integer st n <> 0 holds
a mod n,a are_congruent_mod n
Lm8:
for n being Nat
for a being Integer st n <> 0 holds
ex an being Nat st an,a are_congruent_mod n
Lm9:
for a, b, n, x being Nat st a,b are_congruent_mod n & n <> 0 holds
a |^ x,b |^ x are_congruent_mod n
theorem
theorem
begin
theorem
theorem
Lm10:
for F being commutative Skew-Field
for G being Subgroup of MultGroup F
for n being Nat st 0 < n holds
ex f being Polynomial of F st
( deg f = n & ( for x, xn being Element of F
for xz being Element of G st x = xz & xn = xz |^ n holds
eval (f,x) = xn - (1. F) ) )
Lm11:
for F being commutative Skew-Field
for G being Subgroup of MultGroup F
for a, b being Element of G
for n being Nat st G is finite & 0 < n & ord a = n & b |^ n = 1_ G holds
b is Element of (gr {a})
theorem