Skip to content

Commit

Permalink
Add Ord,Eq instance to WithFC
Browse files Browse the repository at this point in the history
  • Loading branch information
andrevidela committed Dec 1, 2024
1 parent ace3f3c commit d2ea30b
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions libs/base/Language/Reflection/TT.idr
Original file line number Diff line number Diff line change
Expand Up @@ -93,6 +93,16 @@ export
Traversable WithFC where
traverse f (MkFCVal fc val) = map (MkFCVal fc) (f val)

||| Locations are not taken into account when comparing reflected trees
export
Eq a => Eq (WithFC a) where
x == y = x.value == y.value

||| Locations are not taken into account when comparing reflected trees
export
Ord a => Ord (WithFC a) where
compare x y = compare x.value y.value

public export
data NameType : Type where
Bound : NameType
Expand Down

0 comments on commit d2ea30b

Please sign in to comment.