This theory proves that \(\leq\) is a linear order on \(\mathbb{N}\). \(\leq\) is defined in Isabelle's Nat theory, and linear order is defined in Order_ZF theory. Contributed by Seo Sanghyeon.
This is the only section in this theory.
To prove that \(\leq\) is a total order, we use a result on ordinals.
lemma NatOrder_ZF_1_L1:
assumes \( a\in nat \) and \( b\in nat \)
shows \( a \leq b \vee b \leq a \)proof\(\leq\) is antisymmetric, transitive, total, and linear. Proofs by rewrite using definitions.
lemma NatOrder_ZF_1_L2:
shows \( \text{antisym}(Le) \), \( \text{trans}(Le) \), \( Le \text{ is total on } nat \), \( \text{IsLinOrder}(nat,Le) \)proofThe order on natural numbers is linear on every natural number. Recall that each natural number is a subset of the set of all natural numbers (as well as a member).
lemma natord_lin_on_each_nat:
assumes A1: \( n \in nat \)
shows \( \text{IsLinOrder}(n,Le) \)proofassumes \( a\in nat \) and \( b\in nat \)
shows \( a \leq b \vee b \leq a \)assumes \( n \in nat \)
shows \( n \subseteq nat \)assumes \( \text{IsLinOrder}(X,r) \) and \( A\subseteq X \)
shows \( \text{IsLinOrder}(A,r) \) and \( \text{IsLinOrder}(A,r \cap A\times A) \)