begin
theorem
canceled;
theorem
begin
theorem
canceled;
theorem Th4:
theorem
theorem
theorem
for
i,
j,
k,
l being
Nat st
i <= j &
k <= j &
i = (j -' k) + l holds
k = (j -' i) + l
theorem
theorem
for
j,
i being
Nat st
j < i holds
(i -' (j + 1)) + 1
= i -' j
theorem Th10:
for
i,
j being
Nat st
i >= j holds
j -' i = 0
theorem Th11:
theorem Th12:
theorem
theorem Th14:
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
for
n,
k being
Nat st
n <= k &
k < n + n holds
k div n = 1
theorem Th23:
theorem
for
n being
Nat holds
( not
n is
even iff
n mod 2
= 1 )
theorem
theorem Th26:
theorem
theorem
theorem
:: deftheorem Def1 defines trivial NAT_2:def 1 :
for n being Nat holds
( n is trivial iff ( n = 0 or n = 1 ) );
theorem
theorem
scheme
Indfrom2{
P1[
set ] } :
provided
A1:
P1[2]
and A2:
for
k being non
trivial Nat st
P1[
k] holds
P1[
k + 1]
begin
theorem
for
i,
j,
k being
Nat holds
(i -' j) -' k = i -' (j + k)