Skip to content

Commit

Permalink
Add _>>_ for IO.Primitive.Core
Browse files Browse the repository at this point in the history
This has to be in scope for desugaring `do` blocks that don't bind
intermediate results.
  • Loading branch information
ncfavier committed May 1, 2024
1 parent ea994a0 commit f7c78e8
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 0 deletions.
5 changes: 5 additions & 0 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -492,6 +492,11 @@ Additions to existing modules
forever : IO ⊤ → IO ⊤
```

* In `IO.Primitive.Core`:
```agda
_>>_ : IO A → IO B → IO B
```

* In `Data.Word.Base`:
```agda
_≤_ : Rel Word64 zero
Expand Down
3 changes: 3 additions & 0 deletions src/IO/Primitive/Core.agda
Original file line number Diff line number Diff line change
Expand Up @@ -36,3 +36,6 @@ postulate
-- Haskell-style alternative syntax
return : A IO A
return = pure

_>>_ : IO A IO B IO B
a >> b = a >>= λ _ b

0 comments on commit f7c78e8

Please sign in to comment.