begin
theorem Th1:
theorem Th2:
theorem Th3:
Lm1:
for a being Integer holds
( a divides - a & - a divides a )
Lm2:
for a, b, c being Integer st a divides b & b divides c holds
a divides c
Lm3:
for a, b being Integer holds
( a divides b iff a divides - b )
Lm4:
for a, b being Integer holds
( a divides b iff - a divides b )
Lm5:
for a being Integer holds
( a divides 0 & 1 divides a & - 1 divides a )
Lm6:
for a, b, c being Integer st a divides b & a divides c holds
a divides b mod c
Lm7:
for k, l being Nat holds
( k divides l iff ex t being Nat st l = k * t )
Lm8:
for i, j being Nat st i divides j & j divides i holds
i = j
:: deftheorem INT_2:def 1 :
canceled;
:: deftheorem Def2 defines lcm INT_2:def 2 :
for a, b being Integer
for b3 being Nat holds
( b3 = a lcm b iff ( a divides b3 & b divides b3 & ( for m being Integer st a divides m & b divides m holds
b3 divides m ) ) );
theorem Th4:
Lm9:
for j, i being Nat st 0 < j & i divides j holds
i <= j
:: deftheorem Def3 defines gcd INT_2:def 3 :
for a, b being Integer
for b3 being Nat holds
( b3 = a gcd b iff ( b3 divides a & b3 divides b & ( for m being Integer st m divides a & m divides b holds
m divides b3 ) ) );
theorem Th5:
theorem
canceled;
theorem
canceled;
theorem Th8:
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem Th14:
theorem
theorem
theorem Th17:
theorem
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem Th31:
theorem
canceled;
theorem
:: deftheorem Def4 defines are_relative_prime INT_2:def 4 :
for a, b being Integer holds
( a,b are_relative_prime iff a gcd b = 1 );
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem Th39:
theorem Th40:
theorem
:: deftheorem Def5 defines prime INT_2:def 5 :
for p being natural number holds
( p is prime iff ( p > 1 & ( for n being natural number holds
( not n divides p or n = 1 or n = p ) ) ) );
theorem
canceled;
theorem Th43:
theorem Th44:
theorem
canceled;
theorem Th46:
theorem
theorem
begin
theorem
theorem
theorem