Skip to content

Commit

Permalink
WIP: fix rebase with full history unhidding
Browse files Browse the repository at this point in the history
  • Loading branch information
GulinSS committed Nov 28, 2024
1 parent 583157c commit b08c6cc
Showing 1 changed file with 0 additions and 8 deletions.
8 changes: 0 additions & 8 deletions src/Core/Core.idr
Original file line number Diff line number Diff line change
Expand Up @@ -855,14 +855,6 @@ namespace SnocList
traverseFC : (a -> Core b) -> WithFC a -> Core (WithFC b)
traverseFC f (MkFCVal fc x) = MkFCVal fc <$> f x

namespace SnocList
export
traverse_ : (a -> Core b) -> SnocList a -> Core ()
traverse_ f [<] = pure ()
traverse_ f (xs :< x)
= Core.do ignore (f x)
traverse_ f xs

namespace PiInfo
export
traverse : (a -> Core b) -> PiInfo a -> Core (PiInfo b)
Expand Down

0 comments on commit b08c6cc

Please sign in to comment.