mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 08:11:45 +03:00
22 lines
328 B
Idris
22 lines
328 B
Idris
module Data.Binary.Digit
|
|
|
|
%default total
|
|
|
|
||| This is essentially Bool but with names that are easier
|
|
||| to understand
|
|
public export
|
|
data Digit : Type where
|
|
O : Digit
|
|
I : Digit
|
|
|
|
||| Translation to Bool
|
|
public export
|
|
isI : Digit -> Bool
|
|
isI I = True
|
|
isI O = False
|
|
|
|
public export
|
|
toNat : Digit -> Nat
|
|
toNat O = 0
|
|
toNat I = 1
|