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

definition
mode Nat is Element of NAT ;
end;

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

theorem Th2: :: NAT_1:2  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for X being Subset of REAL st 0 in X & ( for x being Real st x in X holds
x + 1 in X ) holds
for k being Nat holds k in X
proof end;

definition
let n, k be Nat;
:: original: +
redefine func n + k -> Nat;
coherence
n + k is Nat
proof end;
end;

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

scheme :: NAT_1:sch 1
Ind{ P1[ Nat] } :
for k being Nat holds P1[k]
provided
A1: P1[0] and
A2: for k being Nat st P1[k] holds
P1[k + 1]
proof end;

scheme :: NAT_1:sch 2
NatInd{ P1[ natural number ] } :
for k being natural number holds P1[k]
provided
A1: P1[0] and
A2: for k being natural number st P1[k] holds
P1[k + 1]
proof end;

definition
let n, k be Nat;
:: original: *
redefine func n * k -> Nat;
coherence
n * k is Nat
proof end;
end;

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

theorem Th18: :: NAT_1:18  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i being natural number holds 0 <= i
proof end;

theorem :: NAT_1:19  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i being natural number st 0 <> i holds
0 < i by Th18;

theorem Th20: :: NAT_1:20  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j, h being natural number st i <= j holds
i * h <= j * h
proof end;

theorem :: NAT_1:21  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i being natural number holds 0 < i + 1
proof end;

theorem Th22: :: NAT_1:22  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i being natural number holds
( i = 0 or ex k being Nat st i = k + 1 )
proof end;

theorem Th23: :: NAT_1:23  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number st i + j = 0 holds
( i = 0 & j = 0 )
proof end;

registration
cluster non zero natural set ;
existence
not for b1 being natural number holds b1 is empty
proof end;
end;

registration
let m be natural number ;
let n be non zero natural number ;
cluster m + n -> non zero natural ;
coherence
not m + n is empty
by Th23;
cluster n + m -> non zero natural ;
coherence
not n + m is empty
;
end;

scheme :: NAT_1:sch 3
DefbyInd{ F1() -> Nat, F2( Nat, Nat) -> Nat, P1[ Nat, Nat] } :
( ( for k being Nat ex n being Nat st P1[k,n] ) & ( for k, n, m being Nat st P1[k,n] & P1[k,m] holds
n = m ) )
provided
A1: for k, n being Nat holds
( P1[k,n] iff ( ( k = 0 & n = F1() ) or ex m, l being Nat st
( k = m + 1 & P1[m,l] & n = F2(k,l) ) ) )
proof end;

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

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

theorem Th26: :: NAT_1:26  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number holds
( not i <= j + 1 or i <= j or i = j + 1 )
proof end;

theorem :: NAT_1:27  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number st i <= j & j <= i + 1 & not i = j holds
j = i + 1
proof end;

theorem Th28: :: NAT_1:28  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number st i <= j holds
ex k being Nat st j = i + k
proof end;

theorem Th29: :: NAT_1:29  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number holds i <= i + j
proof end;

scheme :: NAT_1:sch 4
CompInd{ P1[ Nat] } :
for k being Nat holds P1[k]
provided
A1: for k being Nat st ( for n being Nat st n < k holds
P1[n] ) holds
P1[k]
proof end;

scheme :: NAT_1:sch 5
Min{ P1[ Nat] } :
ex k being Nat st
( P1[k] & ( for n being Nat st P1[n] holds
k <= n ) )
provided
A1: ex k being Nat st P1[k]
proof end;

scheme :: NAT_1:sch 6
Max{ P1[ Nat], F1() -> Nat } :
ex k being Nat st
( P1[k] & ( for n being Nat st P1[n] holds
n <= k ) )
provided
A1: for k being Nat st P1[k] holds
k <= F1() and
A2: ex k being Nat st P1[k]
proof end;

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

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

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

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

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

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

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

theorem Th37: :: NAT_1:37  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j, h being natural number st i <= j holds
i <= j + h
proof end;

theorem Th38: :: NAT_1:38  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number holds
( i < j + 1 iff i <= j )
proof end;

theorem Th39: :: NAT_1:39  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for j being natural number st j < 1 holds
j = 0
proof end;

theorem Th40: :: NAT_1:40  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number st i * j = 1 holds
( i = 1 & j = 1 )
proof end;

theorem Th41: :: NAT_1:41  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, n being natural number st k <> 0 holds
n < n + k
proof end;

scheme :: NAT_1:sch 7
Regr{ P1[ Nat] } :
P1[0]
provided
A1: ex k being Nat st P1[k] and
A2: for k being Nat st k <> 0 & P1[k] holds
ex n being Nat st
( n < k & P1[n] )
proof end;

theorem Th42: :: NAT_1:42  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for m being Nat st 0 < m holds
for n being Nat ex k, t being Nat st
( n = (m * k) + t & t < m )
proof end;

theorem Th43: :: NAT_1:43  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, m, k, k1, t, t1 being natural number st n = (m * k) + t & t < m & n = (m * k1) + t1 & t1 < m holds
( k = k1 & t = t1 )
proof end;

definition
let k, l be natural number ;
A1: ( k is Nat & l is Nat ) by ORDINAL2:def 21;
func k div l -> Nat means :Def1: :: NAT_1:def 1
( ex t being Nat st
( k = (l * it) + t & t < l ) or ( it = 0 & l = 0 ) );
existence
ex b1 being Nat st
( ex t being Nat st
( k = (l * b1) + t & t < l ) or ( b1 = 0 & l = 0 ) )
proof end;
uniqueness
for b1, b2 being Nat st ( ex t being Nat st
( k = (l * b1) + t & t < l ) or ( b1 = 0 & l = 0 ) ) & ( ex t being Nat st
( k = (l * b2) + t & t < l ) or ( b2 = 0 & l = 0 ) ) holds
b1 = b2
proof end;
func k mod l -> Nat means :Def2: :: NAT_1:def 2
( ex t being Nat st
( k = (l * t) + it & it < l ) or ( it = 0 & l = 0 ) );
existence
ex b1 being Nat st
( ex t being Nat st
( k = (l * t) + b1 & b1 < l ) or ( b1 = 0 & l = 0 ) )
proof end;
uniqueness
for b1, b2 being Nat st ( ex t being Nat st
( k = (l * t) + b1 & b1 < l ) or ( b1 = 0 & l = 0 ) ) & ( ex t being Nat st
( k = (l * t) + b2 & b2 < l ) or ( b2 = 0 & l = 0 ) ) holds
b1 = b2
proof end;
end;

:: deftheorem Def1 defines div NAT_1:def 1 :
for k, l being natural number
for b3 being Nat holds
( b3 = k div l iff ( ex t being Nat st
( k = (l * b3) + t & t < l ) or ( b3 = 0 & l = 0 ) ) );

:: deftheorem Def2 defines mod NAT_1:def 2 :
for k, l being natural number
for b3 being Nat holds
( b3 = k mod l iff ( ex t being Nat st
( k = (l * t) + b3 & b3 < l ) or ( b3 = 0 & l = 0 ) ) );

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

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

theorem Th46: :: NAT_1:46  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number st 0 < i holds
j mod i < i
proof end;

theorem Th47: :: NAT_1:47  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number st 0 < i holds
j = (i * (j div i)) + (j mod i)
proof end;

definition
let k, l be natural number ;
pred k divides l means :Def3: :: NAT_1:def 3
ex t being Nat st l = k * t;
reflexivity
for k being natural number ex t being Nat st k = k * t
proof end;
end;

:: deftheorem Def3 defines divides NAT_1:def 3 :
for k, l being natural number holds
( k divides l iff ex t being Nat st l = k * t );

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

theorem Th49: :: NAT_1:49  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for j, i being natural number holds
( j divides i iff i = j * (i div j) )
proof end;

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

theorem :: NAT_1:51  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j, h being natural number st i divides j & j divides h holds
i divides h
proof end;

theorem Th52: :: NAT_1:52  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j being natural number st i divides j & j divides i holds
i = j
proof end;

theorem Th53: :: NAT_1:53  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i being natural number holds
( i divides 0 & 1 divides i )
proof end;

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

theorem Th55: :: NAT_1:55  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j, h being natural number st i divides j & i divides h holds
i divides j + h
proof end;

theorem Th56: :: NAT_1:56  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j, h being natural number st i divides j holds
i divides j * h
proof end;

theorem Th57: :: NAT_1:57  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j, h being natural number st i divides j & i divides j + h holds
i divides h
proof end;

theorem Th58: :: NAT_1:58  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for i, j, h being natural number st i divides j & i divides h holds
i divides j mod h
proof end;

definition
let k, n be Nat;
func k lcm n -> Nat means :Def4: :: NAT_1:def 4
( k divides it & n divides it & ( for m being Nat st k divides m & n divides m holds
it divides m ) );
existence
ex b1 being Nat st
( k divides b1 & n divides b1 & ( for m being Nat st k divides m & n divides m holds
b1 divides m ) )
proof end;
uniqueness
for b1, b2 being Nat st k divides b1 & n divides b1 & ( for m being Nat st k divides m & n divides m holds
b1 divides m ) & k divides b2 & n divides b2 & ( for m being Nat st k divides m & n divides m holds
b2 divides m ) holds
b1 = b2
proof end;
idempotence
for k being Nat holds
( k divides k & k divides k & ( for m being Nat st k divides m & k divides m holds
k divides m ) )
;
commutativity
for b1, k, n being Nat st k divides b1 & n divides b1 & ( for m being Nat st k divides m & n divides m holds
b1 divides m ) holds
( n divides b1 & k divides b1 & ( for m being Nat st n divides m & k divides m holds
b1 divides m ) )
;
end;

:: deftheorem Def4 defines lcm NAT_1:def 4 :
for k, n, b3 being Nat holds
( b3 = k lcm n iff ( k divides b3 & n divides b3 & ( for m being Nat st k divides m & n divides m holds
b3 divides m ) ) );

definition
let k, n be Nat;
func k hcf n -> Nat means :Def5: :: NAT_1:def 5
( it divides k & it divides n & ( for m being Nat st m divides k & m divides n holds
m divides it ) );
existence
ex b1 being Nat st
( b1 divides k & b1 divides n & ( for m being Nat st m divides k & m divides n holds
m divides b1 ) )
proof end;
uniqueness
for b1, b2 being Nat st b1 divides k & b1 divides n & ( for m being Nat st m divides k & m divides n holds
m divides b1 ) & b2 divides k & b2 divides n & ( for m being Nat st m divides k & m divides n holds
m divides b2 ) holds
b1 = b2
proof end;
idempotence
for k being Nat holds
( k divides k & k divides k & ( for m being Nat st m divides k & m divides k holds
m divides k ) )
;
commutativity
for b1, k, n being Nat st b1 divides k & b1 divides n & ( for m being Nat st m divides k & m divides n holds
m divides b1 ) holds
( b1 divides n & b1 divides k & ( for m being Nat st m divides n & m divides k holds
m divides b1 ) )
;
end;

:: deftheorem Def5 defines hcf NAT_1:def 5 :
for k, n, b3 being Nat holds
( b3 = k hcf n iff ( b3 divides k & b3 divides n & ( for m being Nat st m divides k & m divides n holds
m divides b3 ) ) );

scheme :: NAT_1:sch 8
Euklides{ F1( Nat) -> Nat, F2() -> Nat, F3() -> Nat } :
ex n being Nat st
( F1(n) = F2() hcf F3() & F1((n + 1)) = 0 )
provided
A1: ( 0 < F3() & F3() < F2() ) and
A2: ( F1(0) = F2() & F1(1) = F3() ) and
A3: for n being Nat holds F1((n + 2)) = F1(n) mod F1((n + 1))
proof end;

registration
cluster -> ordinal Element of NAT ;
coherence
for b1 being Nat holds b1 is ordinal
;
end;

registration
cluster non empty ordinal Element of K40(REAL );
existence
ex b1 being Subset of REAL st
( not b1 is empty & b1 is ordinal )
proof end;
end;

theorem :: NAT_1:59  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, n being natural number holds
( k < k + n iff 1 <= n )
proof end;

theorem :: NAT_1:60  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, n being natural number st k < n holds
n - 1 is Nat
proof end;

theorem Th61: :: NAT_1:61  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, n being natural number st k <= n holds
n - k is Nat
proof end;

theorem :: NAT_1:62  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n being natural number holds
( n mod 2 = 0 or n mod 2 = 1 )
proof end;

theorem :: NAT_1:63  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, n being natural number holds (k * n) mod k = 0
proof end;

theorem :: NAT_1:64  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, l being natural number st k > 1 holds
1 mod k = 1
proof end;

theorem :: NAT_1:65  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, l, n, m being natural number st k mod n = 0 & l = k - (m * n) holds
l mod n = 0
proof end;

theorem :: NAT_1:66  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, l, n being natural number st n <> 0 & k mod n = 0 & l < n holds
(k + l) mod n = l
proof end;

theorem :: NAT_1:67  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, l, n being natural number st k mod n = 0 holds
(k + l) mod n = l mod n
proof end;

theorem :: NAT_1:68  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, n being natural number st k <> 0 holds
(k * n) div k = n
proof end;

theorem :: NAT_1:69  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for k, n, l being natural number st k mod n = 0 holds
(k + l) div n = (k div n) + (l div n)
proof end;

theorem Th70: :: NAT_1:70  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
( not m < n + 1 or m < n or m = n )
proof end;

theorem :: NAT_1:71  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
( not k < 2 or k = 0 or k = 1 )
proof end;

registration
cluster non zero Element of NAT ;
existence
not for b1 being Nat holds b1 is empty
proof end;
end;

registration
cluster -> ordinal non negative Element of NAT ;
coherence
for b1 being Element of NAT holds not b1 is negative
by Th18;
end;

registration
cluster natural -> natural non negative set ;
coherence
for b1 being natural number holds not b1 is negative
by Th18;
end;

theorem :: NAT_1:72  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 <> 0 holds
(m * k) div k = m
proof end;

theorem Th1: :: NAT_1:73  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 natural number holds m mod n = ((n * k) + m) mod n
proof end;

theorem Th2: :: NAT_1:74  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for p, s, n being natural number holds (p + s) mod n = ((p mod n) + s) mod n
proof end;

theorem :: NAT_1:75  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for p, s, n being natural number holds (p + s) mod n = (p + (s mod n)) mod n by Th2;

theorem Th4: :: NAT_1:76  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n, k being natural number st k < n holds
k mod n = k
proof end;

theorem Th5: :: NAT_1:77  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n being natural number holds n mod n = 0
proof end;

theorem Th6: :: NAT_1:78  Show TPTP formulae Show IDV graph:: Showing IDV graph ... (Click the Palm Tree again to close it) Show TPTP problem
for n being natural number holds 0 = 0 mod n
proof end;