Skip to content

Commit

Permalink
rename val to value
Browse files Browse the repository at this point in the history
  • Loading branch information
andrevidela committed Nov 24, 2024
1 parent 471e473 commit a49d771
Show file tree
Hide file tree
Showing 2 changed files with 7 additions and 7 deletions.
6 changes: 3 additions & 3 deletions libs/base/Language/Reflection/TT.idr
Original file line number Diff line number Diff line change
Expand Up @@ -74,7 +74,7 @@ public export
record WithFC (ty : Type) where
constructor MkFCVal
fc : FC
val : ty
value : ty

||| Smart constructor for WithFC that uses EmptyFC as location
%inline export
Expand All @@ -83,11 +83,11 @@ NoFC = MkFCVal EmptyFC

export
Functor WithFC where
map f = { val $= f}
map f = { value $= f}

export
Foldable WithFC where
foldr f i v = f v.val i
foldr f i v = f v.value i

export
Traversable WithFC where
Expand Down
8 changes: 4 additions & 4 deletions libs/base/Language/Reflection/TTImp.idr
Original file line number Diff line number Diff line change
Expand Up @@ -415,7 +415,7 @@ parameters {auto eqTTImp : Eq TTImp}

public export
Eq ITy where
MkTy _ n ty == MkTy _ n' ty' = n.val == n'.val && ty == ty'
MkTy _ n ty == MkTy _ n' ty' = n.value == n'.value && ty == ty'

public export
Eq Data where
Expand All @@ -442,7 +442,7 @@ parameters {auto eqTTImp : Eq TTImp}

public export
Eq Decl where
IClaim c == IClaim c' = c.val == c'.val
IClaim c == IClaim c' = c.value == c'.value
IData _ v t d == IData _ v' t' d' =
v == v' && t == t' && d == d'
IDef _ n cs == IDef _ n' cs' =
Expand Down Expand Up @@ -552,7 +552,7 @@ mutual

public export
Show ITy where
show (MkTy fc n ty) = "\{show n.val} : \{show ty}"
show (MkTy fc n ty) = "\{show n.value} : \{show ty}"

Show IClaimData where
show (MkIClaimData rig vis xs sig)
Expand All @@ -561,7 +561,7 @@ mutual

public export
Show Decl where
show (IClaim claim) = show claim.val
show (IClaim claim) = show claim.value
show (IData fc vis treq dt)
= unwords [ show vis
, showTotalReq treq (show dt)
Expand Down

0 comments on commit a49d771

Please sign in to comment.