Skip to content

Commit

Permalink
remove TelNames
Browse files Browse the repository at this point in the history
  • Loading branch information
andrevidela committed Jan 17, 2025
1 parent d1801f3 commit d55cf68
Showing 1 changed file with 0 additions and 13 deletions.
13 changes: 0 additions & 13 deletions src/Core/TT/Term.idr
Original file line number Diff line number Diff line change
Expand Up @@ -557,19 +557,6 @@ covering
assert_total (showSep " " (map show args))
++ ")"

||| A telescope of names and their associated types/terms
public export
data TelNames : List Name -> Type where
Nil : TelNames xs
AddName : (n : Name) -> Term vars -> (isImplicit : Bool) -> TelNames (n :: vars) -> TelNames vars

covering export
{vars : _} -> Show (TelNames vars) where
show [] = ""
show (AddName n ty _ []) = "(\{show n} : \{show ty})"
show (AddName n ty False rest) = "(\{show n} : \{show ty}) -> \{show rest}"
show (AddName n ty True rest) = "{\{show n} : \{show ty}} -> \{show rest}"

||| Obtain the telescope of names and their types
export
collectPiNames : Term vars -> List (Bool, Name)
Expand Down

0 comments on commit d55cf68

Please sign in to comment.