The naturals are defined as a set of objects which obey the following axioms:
0 is natural.
If n is a natural, then n++ is also natural.
n++=0.
n++=m++ can be rewritten as n=m.
Let P be a proposition over any natural n. If P(0) is true, and if whenever P(n) is true we also have P(n++) is true, then P is true for any natural.
Logical Assumptions
Let a,b,c be naturals.
a=a(reflexive)
a=b⟷b=a(symmetric)
(a=b)∧(b=c)⟶a=c(transitive)
Set Theory with 2nd Order Logic
∃(Ø,N):Ø∈N
∀(n):n∪{n}∈N
∀(n,m):n∪{n}=m∪{m}⟶n=m
∀(n):[P(Ø)∧P(n)→P(n∪{n})]⟶P(n)
Definition 1: Addition
Addition + is a closed binary operator over any pair of naturals (n,m).
{0+m(n++)+m=m=(n+m)++
Proposition 1: n+0=n
We use induction to ask if the proposition P(n)↦n+0=n is true for any natural n.
Base Case
We evaluate the base case P(0) which maps to the proposition 0+0=0.
0+00=?0=✓0
We use the definition of addition to rewrite the left-hand side of the equation to arrive at 0=0, which we know to be reflexively true.
Inductive Case
For any specific n, is assuming P(n) is sufficient to know P(n++)?
(n++)+0(n+0)++n+0=n++=n++=n
The case of P(n++) can be written as P(n). By the inductive axiom we know that P(n) is true for all naturals.
Proposition 2: n+(m++)=(n+m)++
Using induction we ask if P(n)↦n+m++=(n+m)++ is true for any n,m∈N. Informally we are wondering whether we can use a “reversed” rule for addition as a stepping stone to commutativity.
Base Case
0+m++m++=(0+m)++=m++
Inductive Case
(n++)+(m++)=((n++)+m)++(1)
(n+(m++))++=((n+m)++)++(2)
n+(m++)=(n+m)++(3)
This is our inductive hypothesis.
We rewrite the expression on both sides according to definition of addition.
We removed a layer of succession from both sides by the 4th Peano axiom.
This also means that both n,m must be 0 for the expression (n+m=0).
Corollary: Positives have unique predecessor
Argument. For every positive natural n there exists a unique natural a such that n=a++.
Proof. Let’s say there exists another natural b where (b++=n). Then (a++=b++) which implies (a=b). This means all predecessors are unique. Now let’s say that for all positive n we have (n=a++).
P(n):=∃(a):n=a++
P(1)↦1=✓0++
P(n++)↦n++=?a++
n=✓a
Definition: Greater/Lesser or Equal
For any naturals {a,b} the partial order (a≤b) is defined as the proposition that there exists a natural n where (a+n=b) is true.
(a≤b):=∃(n):a+n=b
Since n could be 0 it’s possible that a=b. If n were positive then we know that a=b, which is how we define the strict order operator:
(a<b):=(a≤b)∧(a=b)
This definition can be restated as:
a<ba<b⟶(a+n=b)∧(n=0)⟶a+(n++)=b
Lemma: Trichotemy of the Naturals
For any two naturals {a,b} only one of these statements can be true at a time.
This can be finitely proven through truth tabling.