begin
theorem Th1:
theorem Th2:
Lm1:
for x, y being Integer holds
( ( x divides y implies y mod x = 0 ) & ( x <> 0 & y mod x = 0 implies x divides y ) )
:: deftheorem Def1 defines Poly-INT INT_5:def 1 :
for fp being FinSequence of INT
for b2 being Function of INT,INT holds
( b2 = Poly-INT fp iff for x being Element of INT ex fr being FinSequence of INT st
( len fr = len fp & ( for d being Nat st d in dom fr holds
fr . d = (fp . d) * (x |^ (d -' 1)) ) & b2 . x = Sum fr ) );
theorem Th3:
theorem
theorem Th5:
theorem Th6:
theorem Th7:
theorem Th8:
:: deftheorem Def2 defines is_quadratic_residue_mod INT_5:def 2 :
for a being Integer
for m being Nat holds
( a is_quadratic_residue_mod m iff ex x being Integer st ((x ^2) - a) mod m = 0 );
theorem Th9:
theorem
theorem Th11:
Lm2:
for i being Integer
for p being Prime holds
( i,p are_relative_prime or p divides i )
theorem Th12:
theorem Th13:
theorem Th14:
theorem
theorem Th16:
theorem Th17:
theorem Th18:
theorem Th19:
theorem Th20:
theorem Th21:
theorem
theorem
theorem
:: deftheorem Def3 defines Lege INT_5:def 3 :
for a being Integer
for p being Prime holds
( ( a is_quadratic_residue_mod p & a mod p <> 0 implies Lege (a,p) = 1 ) & ( a is_quadratic_residue_mod p & a mod p = 0 implies Lege (a,p) = 0 ) & ( ( not a is_quadratic_residue_mod p or not a mod p <> 0 ) & ( not a is_quadratic_residue_mod p or not a mod p = 0 ) implies Lege (a,p) = - 1 ) );
theorem Th25:
theorem Th26:
theorem
Lm3:
for a being Integer
for p being Prime st a gcd p = 1 holds
not p divides a
theorem Th28:
theorem
theorem
theorem Th31:
theorem Th32:
theorem Th33:
theorem Th34:
theorem
theorem Th36:
theorem
theorem
begin
theorem Th39:
theorem Th40:
theorem Th41:
theorem Th42:
theorem
theorem
theorem Th45:
theorem Th46:
theorem Th47:
theorem Th48:
Lm4:
for fp being FinSequence of NAT holds Sum fp is Element of NAT
;
theorem Th49:
theorem
theorem