view Paper/src/agda/cmp.agda @ 32:4915eaa51ee0 default tip

Add front
author soto <soto@cr.ie.u-ryukyu.ac.jp>
date Thu, 23 Feb 2023 18:39:56 +0900
parents a72446879486
children
line wrap: on
line source

module cmp where

open import Data.Nat
open import Data.Nat.Properties as NatProp -- <-cmp
open import Relation.Binary

compare_test : ℕ → ℕ → ℕ
compare_test x y with <-cmp x y
... | tri< a ¬b ¬c = y
... | tri≈ ¬a b ¬c = x
... | tri> ¬a ¬b c = x

-- test = compare_test 7 2
-- 7