1 | module Data.Nat.Order.Strict
4 | import Decidable.Order.Strict
9 | Irreflexive Nat LT where
10 | irreflexive {x = S _} (LTESucc prf) =
11 | irreflexive {rel = Nat.LT} prf
14 | Transitive Nat LT where
15 | transitive xy yz = transitive (lteSuccRight xy) yz
18 | StrictPreorder Nat LT where
21 | decLT : (a, b : Nat) -> DecOrdering {lt = LT} a b
22 | decLT 0 0 = DecEQ Refl
23 | decLT 0 (S b) = DecLT (LTESucc LTEZero)
24 | decLT (S a) 0 = DecGT (LTESucc LTEZero)
25 | decLT (S a) (S b) = case decLT a b of
26 | DecLT a_lt_b => DecLT (LTESucc a_lt_b)
27 | DecEQ Refl => DecEQ Refl
28 | DecGT b_lt_a => DecGT (LTESucc b_lt_a)
31 | StrictOrdered Nat LT where