We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
_>>_
IO.Primitive.Core
1 parent 3d54042 commit 618d838Copy full SHA for 618d838
CHANGELOG.md
@@ -492,6 +492,11 @@ Additions to existing modules
492
forever : IO ⊤ → IO ⊤
493
```
494
495
+* In `IO.Primitive.Core`:
496
+ ```agda
497
+ _>>_ : IO A → IO B → IO B
498
+ ```
499
+
500
* In `Data.Word.Base`:
501
```agda
502
_≤_ : Rel Word64 zero
src/IO/Primitive/Core.agda
@@ -36,3 +36,6 @@ postulate
36
-- Haskell-style alternative syntax
37
return : A → IO A
38
return = pure
39
40
+_>>_ : IO A → IO B → IO B
41
+a >> b = a >>= λ _ → b
0 commit comments