:: NEWTON semantic presentation  Show TPTP formulae Show IDV graph for whole article:: Showing IDV graph ... (Click the Palm Trees again to close it)

theorem :: NEWTON:1  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem :: NEWTON:2  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th3: :: NEWTON:3  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for F, G being FinSequence st len F = len G & ( for i being Nat st i in dom F holds
F . i = G . i ) holds
F = G
proof end;

theorem :: NEWTON:4  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th5: :: NEWTON:5  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n being Nat st n >= 1 holds
Seg n = ({1} \/ { k where k is Nat : ( 1 < k & k < n ) } ) \/ {n}
proof end;

theorem Th6: :: NEWTON:6  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for a being real number
for F being FinSequence of REAL holds len (a * F) = len F
proof end;

theorem Th7: :: NEWTON:7  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n being Nat
for a being real number
for G being FinSequence of REAL holds
( n in dom G iff n in dom (a * G) )
proof end;

definition
let i be natural number ;
let x be real number ;
:: original: |->
redefine func i |-> x -> FinSequence of REAL ;
coherence
i |-> x is FinSequence of REAL
proof end;
end;

definition
let x be real number ;
let n be natural number ;
func x |^ n -> set equals :: NEWTON:def 1
Product (n |-> x);
coherence
Product (n |-> x) is set
;
end;

:: deftheorem defines |^ NEWTON:def 1 :
for x being real number
for n being natural number holds x |^ n = Product (n |-> x);

registration
let x be real number ;
let n be natural number ;
cluster x |^ n -> real ;
coherence
x |^ n is real
;
end;

definition
let x be Real;
let n be natural number ;
:: original: |^
redefine func x |^ n -> Real;
coherence
x |^ n is Real
;
end;

theorem :: NEWTON:8  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th9: :: NEWTON:9  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for x being real number holds x |^ 0 = 1 by FINSEQ_2:72, RVSUM_1:124;

theorem Th10: :: NEWTON:10  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for x being real number holds x |^ 1 = x
proof end;

theorem Th11: :: NEWTON:11  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number
for x being real number holds x |^ (s + 1) = (x |^ s) * x
proof end;

registration
let x, n be natural number ;
cluster x |^ n -> natural real ;
coherence
x |^ n is natural
proof end;
end;

theorem :: NEWTON:12  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number
for x, y being real number holds (x * y) |^ s = (x |^ s) * (y |^ s)
proof end;

theorem :: NEWTON:13  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s, t being natural number
for x being real number holds x |^ (s + t) = (x |^ s) * (x |^ t)
proof end;

theorem :: NEWTON:14  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s, t being natural number
for x being real number holds (x |^ s) |^ t = x |^ (s * t)
proof end;

theorem Th15: :: NEWTON:15  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number holds 1 |^ s = 1
proof end;

theorem :: NEWTON:16  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number st s >= 1 holds
0 |^ s = 0
proof end;

definition
let n be natural number ;
:: original: idseq
redefine func idseq n -> FinSequence of REAL ;
coherence
idseq n is FinSequence of REAL
proof end;
end;

definition
let n be natural number ;
func n ! -> set equals :: NEWTON:def 2
Product (idseq n);
coherence
Product (idseq n) is set
;
end;

:: deftheorem defines ! NEWTON:def 2 :
for n being natural number holds n ! = Product (idseq n);

registration
let n be natural number ;
cluster n ! -> real ;
coherence
n ! is real
;
end;

definition
let n be natural number ;
:: original: !
redefine func n ! -> Real;
coherence
n ! is Real
;
end;

theorem :: NEWTON:17  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th18: :: NEWTON:18  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
0 ! = 1 by FINSEQ_2:58, RVSUM_1:124;

theorem Th19: :: NEWTON:19  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
1 ! = 1 by FINSEQ_2:59, RVSUM_1:125;

theorem :: NEWTON:20  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
2 ! = 2
proof end;

theorem Th21: :: NEWTON:21  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number holds (s + 1) ! = (s ! ) * (s + 1)
proof end;

theorem Th22: :: NEWTON:22  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number holds s ! is Nat
proof end;

theorem Th23: :: NEWTON:23  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number holds s ! > 0
proof end;

theorem :: NEWTON:24  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th25: :: NEWTON:25  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s, t being natural number holds (s ! ) * (t ! ) <> 0
proof end;

definition
let k, n be natural number ;
func n choose k -> set means :Def3: :: NEWTON:def 3
for l being natural number st l = n - k holds
it = (n ! ) / ((k ! ) * (l ! )) if n >= k
otherwise it = 0;
consistency
for b1 being set holds verum
;
existence
( ( n >= k implies ex b1 being set st
for l being natural number st l = n - k holds
b1 = (n ! ) / ((k ! ) * (l ! )) ) & ( not n >= k implies ex b1 being set st b1 = 0 ) )
proof end;
uniqueness
for b1, b2 being set holds
( ( n >= k & ( for l being natural number st l = n - k holds
b1 = (n ! ) / ((k ! ) * (l ! )) ) & ( for l being natural number st l = n - k holds
b2 = (n ! ) / ((k ! ) * (l ! )) ) implies b1 = b2 ) & ( not n >= k & b1 = 0 & b2 = 0 implies b1 = b2 ) )
proof end;
end;

:: deftheorem Def3 defines choose NEWTON:def 3 :
for k, n being natural number
for b3 being set holds
( ( n >= k implies ( b3 = n choose k iff for l being natural number st l = n - k holds
b3 = (n ! ) / ((k ! ) * (l ! )) ) ) & ( not n >= k implies ( b3 = n choose k iff b3 = 0 ) ) );

registration
let k, n be natural number ;
cluster n choose k -> real ;
coherence
n choose k is real
proof end;
end;

definition
let k, n be natural number ;
:: original: choose
redefine func n choose k -> Real;
coherence
n choose k is Real
by XREAL_0:def 1;
end;

theorem :: NEWTON:26  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th27: :: NEWTON:27  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
0 choose 0 = 1
proof end;

theorem :: NEWTON:28  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th29: :: NEWTON:29  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number holds s choose 0 = 1
proof end;

theorem Th30: :: NEWTON:30  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s, t being natural number st s >= t holds
for r being natural number st r = s - t holds
s choose t = s choose r
proof end;

theorem Th31: :: NEWTON:31  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number holds s choose s = 1
proof end;

theorem Th32: :: NEWTON:32  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for t, s being natural number holds (t + 1) choose (s + 1) = (t choose (s + 1)) + (t choose s)
proof end;

theorem Th33: :: NEWTON:33  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number st s >= 1 holds
s choose 1 = s
proof end;

theorem :: NEWTON:34  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s, t being natural number st s >= 1 & t = s - 1 holds
s choose t = s
proof end;

theorem :: NEWTON:35  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s, r being natural number holds s choose r is Nat
proof end;

theorem :: NEWTON:36  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m being Nat
for F being FinSequence of REAL st m <> 0 & len F = m & ( for i, l being Nat st i in dom F & l = (n + i) - 1 holds
F . i = l choose n ) holds
Sum F = (n + m) choose (n + 1)
proof end;

definition
let a, b be real number ;
let n be natural number ;
func a,b In_Power n -> FinSequence of REAL means :Def4: :: NEWTON:def 4
( len it = n + 1 & ( for i, l, m being natural number st i in dom it & m = i - 1 & l = n - m holds
it . i = ((n choose m) * (a |^ l)) * (b |^ m) ) );
existence
ex b1 being FinSequence of REAL st
( len b1 = n + 1 & ( for i, l, m being natural number st i in dom b1 & m = i - 1 & l = n - m holds
b1 . i = ((n choose m) * (a |^ l)) * (b |^ m) ) )
proof end;
uniqueness
for b1, b2 being FinSequence of REAL st len b1 = n + 1 & ( for i, l, m being natural number st i in dom b1 & m = i - 1 & l = n - m holds
b1 . i = ((n choose m) * (a |^ l)) * (b |^ m) ) & len b2 = n + 1 & ( for i, l, m being natural number st i in dom b2 & m = i - 1 & l = n - m holds
b2 . i = ((n choose m) * (a |^ l)) * (b |^ m) ) holds
b1 = b2
proof end;
end;

:: deftheorem Def4 defines In_Power NEWTON:def 4 :
for a, b being real number
for n being natural number
for b4 being FinSequence of REAL holds
( b4 = a,b In_Power n iff ( len b4 = n + 1 & ( for i, l, m being natural number st i in dom b4 & m = i - 1 & l = n - m holds
b4 . i = ((n choose m) * (a |^ l)) * (b |^ m) ) ) );

theorem :: NEWTON:37  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th38: :: NEWTON:38  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for a, b being real number holds a,b In_Power 0 = <*1*>
proof end;

theorem Th39: :: NEWTON:39  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number
for a, b being real number holds (a,b In_Power s) . 1 = a |^ s
proof end;

theorem Th40: :: NEWTON:40  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number
for a, b being real number holds (a,b In_Power s) . (s + 1) = b |^ s
proof end;

theorem Th41: :: NEWTON:41  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for a, b being real number
for s being natural number holds (a + b) |^ s = Sum (a,b In_Power s)
proof end;

definition
let n be natural number ;
func Newton_Coeff n -> FinSequence of REAL means :Def5: :: NEWTON:def 5
( len it = n + 1 & ( for i, k being natural number st i in dom it & k = i - 1 holds
it . i = n choose k ) );
existence
ex b1 being FinSequence of REAL st
( len b1 = n + 1 & ( for i, k being natural number st i in dom b1 & k = i - 1 holds
b1 . i = n choose k ) )
proof end;
uniqueness
for b1, b2 being FinSequence of REAL st len b1 = n + 1 & ( for i, k being natural number st i in dom b1 & k = i - 1 holds
b1 . i = n choose k ) & len b2 = n + 1 & ( for i, k being natural number st i in dom b2 & k = i - 1 holds
b2 . i = n choose k ) holds
b1 = b2
proof end;
end;

:: deftheorem Def5 defines Newton_Coeff NEWTON:def 5 :
for n being natural number
for b2 being FinSequence of REAL holds
( b2 = Newton_Coeff n iff ( len b2 = n + 1 & ( for i, k being natural number st i in dom b2 & k = i - 1 holds
b2 . i = n choose k ) ) );

theorem :: NEWTON:42  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem Th43: :: NEWTON:43  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number holds Newton_Coeff s = 1,1 In_Power s
proof end;

theorem :: NEWTON:44  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for s being natural number holds 2 |^ s = Sum (Newton_Coeff s)
proof end;

theorem Th45: :: NEWTON:45  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for l, k being Nat st l >= 1 holds
k * l >= k
proof end;

theorem Th46: :: NEWTON:46  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for l, n, k being Nat st l >= 1 & n >= k * l holds
n >= k
proof end;

definition
let n be Nat;
:: original: !
redefine func n ! -> Nat;
coherence
n ! is Nat
by Th22;
end;

theorem Th47: :: NEWTON:47  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for l being Nat st l <> 0 holds
l divides l !
proof end;

theorem :: NEWTON:48  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n being Nat st n <> 0 holds
(n + 1) / n > 1
proof end;

theorem Th49: :: NEWTON:49  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k being Nat holds k / (k + 1) < 1
proof end;

theorem Th50: :: NEWTON:50  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for l being Nat holds l ! >= l
proof end;

theorem Th51: :: NEWTON:51  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being Nat st m <> 1 & m divides n holds
not m divides n + 1
proof end;

theorem :: NEWTON:52  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for l, j being Nat holds
( ( j divides l & j divides l + 1 ) iff j = 1 ) by Th51, NAT_1:53;

theorem Th53: :: NEWTON:53  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, j being Nat st j <> 0 holds
j divides (j + k) !
proof end;

theorem Th54: :: NEWTON:54  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for l, j being Nat st j <= l & j <> 0 holds
j divides l !
proof end;

theorem Th55: :: NEWTON:55  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for l, j being Nat st j <> 1 & j <> 0 & j divides (l ! ) + 1 holds
j > l
proof end;

theorem :: NEWTON:56  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n, k being Nat holds m lcm (n lcm k) = (m lcm n) lcm k
proof end;

theorem Th57: :: NEWTON:57  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being Nat holds
( m divides n iff m lcm n = n )
proof end;

theorem :: NEWTON:58  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m, k being Nat holds
( ( n divides m & k divides m ) iff n lcm k divides m )
proof end;

theorem :: NEWTON:59  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m being Nat holds m lcm 1 = m
proof end;

theorem Th60: :: NEWTON:60  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being Nat holds m lcm n divides m * n
proof end;

theorem :: NEWTON:61  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n, k being Nat holds m hcf (n hcf k) = (m hcf n) hcf k
proof end;

theorem Th62: :: NEWTON:62  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m being Nat st n divides m holds
n hcf m = n
proof end;

theorem :: NEWTON:63  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n, k being Nat holds
( ( m divides n & m divides k ) iff m divides n hcf k )
proof end;

theorem :: NEWTON:64  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m being Nat holds m hcf 1 = 1
proof end;

theorem :: NEWTON:65  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m being Nat holds m hcf 0 = m
proof end;

theorem Th66: :: NEWTON:66  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being Nat holds (m hcf n) lcm n = n
proof end;

theorem Th67: :: NEWTON:67  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being Nat holds m hcf (m lcm n) = m
proof end;

theorem :: NEWTON:68  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being Nat holds m hcf (m lcm n) = (n hcf m) lcm m
proof end;

theorem :: NEWTON:69  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n, k being Nat st m divides n holds
m hcf k divides n hcf k
proof end;

theorem :: NEWTON:70  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n, k being Nat st m divides n holds
k hcf m divides k hcf n
proof end;

theorem :: NEWTON:71  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m being Nat st n > 0 holds
n hcf m > 0
proof end;

theorem :: NEWTON:72  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
canceled;

theorem :: NEWTON:73  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being Nat st m > 0 & n > 0 holds
m lcm n > 0
proof end;

theorem :: NEWTON:74  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m, k being Nat holds (n hcf m) lcm (n hcf k) divides n hcf (m lcm k)
proof end;

theorem :: NEWTON:75  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, l, n being Nat st m divides l holds
m lcm (n hcf l) divides (m lcm n) hcf l
proof end;

theorem :: NEWTON:76  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m being Nat holds n hcf m divides n lcm m
proof end;

theorem :: NEWTON:77  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m being Nat st 0 < m holds
n mod m = n - (m * (n div m))
proof end;

theorem Th78: :: NEWTON:78  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i2, i1 being Integer st i2 >= 0 holds
i1 mod i2 >= 0
proof end;

theorem Th79: :: NEWTON:79  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i2, i1 being Integer st i2 > 0 holds
i1 mod i2 < i2
proof end;

theorem Th80: :: NEWTON:80  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i2, i1 being Integer st i2 <> 0 holds
i1 = ((i1 div i2) * i2) + (i1 mod i2)
proof end;

theorem :: NEWTON:81  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being Nat st ( m > 0 or n > 0 ) holds
ex i, i1 being Integer st (i * m) + (i1 * n) = m hcf n
proof end;

definition
func SetPrimes -> Subset of NAT means :Def6: :: NEWTON:def 6
for n being Nat holds
( n in it iff n is prime );
existence
ex b1 being Subset of NAT st
for n being Nat holds
( n in b1 iff n is prime )
proof end;
uniqueness
for b1, b2 being Subset of NAT st ( for n being Nat holds
( n in b1 iff n is prime ) ) & ( for n being Nat holds
( n in b2 iff n is prime ) ) holds
b1 = b2
proof end;
end;

:: deftheorem Def6 defines SetPrimes NEWTON:def 6 :
for b1 being Subset of NAT holds
( b1 = SetPrimes iff for n being Nat holds
( n in b1 iff n is prime ) );

registration
cluster prime Element of NAT ;
existence
ex b1 being Nat st b1 is prime
by INT_2:44;
end;

definition
mode Prime is prime Nat;
end;

definition
let p be Nat;
func SetPrimenumber p -> Subset of NAT means :Def7: :: NEWTON:def 7
for q being Nat holds
( q in it iff ( q < p & q is prime ) );
existence
ex b1 being Subset of NAT st
for q being Nat holds
( q in b1 iff ( q < p & q is prime ) )
proof end;
uniqueness
for b1, b2 being Subset of NAT st ( for q being Nat holds
( q in b1 iff ( q < p & q is prime ) ) ) & ( for q being Nat holds
( q in b2 iff ( q < p & q is prime ) ) ) holds
b1 = b2
proof end;
end;

:: deftheorem Def7 defines SetPrimenumber NEWTON:def 7 :
for p being Nat
for b2 being Subset of NAT holds
( b2 = SetPrimenumber p iff for q being Nat holds
( q in b2 iff ( q < p & q is prime ) ) );

theorem Th82: :: NEWTON:82  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for p being Nat holds SetPrimenumber p c= SetPrimes
proof end;

theorem :: NEWTON:83  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for p, q being Nat st p < q holds
SetPrimenumber p c= SetPrimenumber q
proof end;

theorem Th84: :: NEWTON:84  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for p being Nat holds SetPrimenumber p c= Seg p
proof end;

theorem :: NEWTON:85  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for p being Nat holds SetPrimenumber p is finite
proof end;

Lm1: for k being Nat holds
( k = 0 or k = 1 or 2 <= k )
proof end;

theorem Th86: :: NEWTON:86  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for l being Nat ex p being Prime st
( p is prime & p > l )
proof end;

theorem :: NEWTON:87  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
SetPrimes <> {} by Def6, INT_2:44;

theorem Th88: :: NEWTON:88  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
{ k where k is Nat : ( k < 2 & k is prime ) } = {}
proof end;

theorem :: NEWTON:89  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for p being Prime holds { k where k is Nat : ( k < p & k is prime ) } c= NAT
proof end;

theorem Th90: :: NEWTON:90  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m being Nat holds { k where k is Nat : ( k < m & k is prime ) } c= Seg m
proof end;

theorem Th91: :: NEWTON:91  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m being Nat holds { k where k is Nat : ( k < m & k is prime ) } is finite
proof end;

theorem Th92: :: NEWTON:92  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for f being Nat holds not f in { k where k is Nat : ( k < f & k is prime ) }
proof end;

theorem :: NEWTON:93  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for f being Nat holds { k where k is Nat : ( k < f & k is prime ) } \/ {f} is finite
proof end;

theorem Th94: :: NEWTON:94  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for f, g being Prime st f < g holds
{ k1 where k1 is Nat : ( k1 < f & k1 is prime ) } \/ {f} c= { k2 where k2 is Nat : ( k2 < g & k2 is prime ) }
proof end;

theorem :: NEWTON:95  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, k being Nat st k > m holds
not k in { k1 where k1 is Nat : ( k1 < m & k1 is prime ) }
proof end;

definition
let n be Nat;
func primenumber n -> Prime means :Def8: :: NEWTON:def 8
ex B being finite set st
( B = { k where k is Nat : ( k < it & k is prime ) } & n = card B );
existence
ex b1 being Prime ex B being finite set st
( B = { k where k is Nat : ( k < b1 & k is prime ) } & n = card B )
proof end;
uniqueness
for b1, b2 being Prime st ex B being finite set st
( B = { k where k is Nat : ( k < b1 & k is prime ) } & n = card B ) & ex B being finite set st
( B = { k where k is Nat : ( k < b2 & k is prime ) } & n = card B ) holds
b1 = b2
proof end;
end;

:: deftheorem Def8 defines primenumber NEWTON:def 8 :
for n being Nat
for b2 being Prime holds
( b2 = primenumber n iff ex B being finite set st
( B = { k where k is Nat : ( k < b2 & k is prime ) } & n = card B ) );

theorem Th96: :: NEWTON:96  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for p being Prime holds SetPrimenumber p = { k where k is Nat : ( k < p & k is prime ) }
proof end;

theorem Th97: :: NEWTON:97  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
not SetPrimes is finite
proof end;

registration
cluster SetPrimes -> non empty infinite ;
coherence
( not SetPrimes is empty & not SetPrimes is finite )
by Th97;
end;

Lm2: for n being Nat st n is prime holds
n > 0
by INT_2:def 5;

theorem :: NEWTON:98  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i being Nat st i is prime holds
for m, n being Nat holds
( not i divides m * n or i divides m or i divides n )
proof end;

theorem :: NEWTON:99  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m being Nat holds m |^ n is Nat
proof end;

theorem :: NEWTON:100  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for x being real number holds
( x |^ 2 = x * x & x ^2 = x |^ 2 )
proof end;

theorem :: NEWTON:101  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m, n being natural number holds
( m div n = m div n & m mod n = m mod n )
proof end;