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.
If \(a,b\) are natural numbers then \(a\) is less or equal \(b\) or \(b\) is (strictly) less than \(a\). We use a result on ordinals in the proof.
lemma nat_order_2cases:
assumes \( a\in nat \) and \( b\in nat \)
shows \( a \leq b \vee b \lt a \)proofA special case of nat_order_2cases: If \(a,b\) are natural numbers then \(a\) is less or equal \(b\) or \(b\) is less or equal than \(a\).
lemma NatOrder_ZF_1_L1:
assumes \( a\in nat \) and \( b\in nat \)
shows \( a \leq b \vee b \leq a \) using assms, nat_order_2cases, leI\(\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 \lt a \)assumes \( 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) \)