mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-29 03:24:02 +03:00
[ refactor ] renamed value to runConst
This commit is contained in:
parent
7863636490
commit
0858c26dcf
@ -6,15 +6,15 @@ import Data.Bits
|
||||
public export
|
||||
record Const (a : Type) (b : Type) where
|
||||
constructor MkConst
|
||||
value : a
|
||||
runConst : a
|
||||
|
||||
public export
|
||||
Eq a => Eq (Const a b) where
|
||||
(==) = (==) `on` value
|
||||
(==) = (==) `on` runConst
|
||||
|
||||
public export
|
||||
Ord a => Ord (Const a b) where
|
||||
compare = compare `on` value
|
||||
compare = compare `on` runConst
|
||||
|
||||
export
|
||||
Show a => Show (Const a b) where
|
||||
|
Loading…
Reference in New Issue
Block a user