A RetroSearch Logo

Home - News ( United States | United Kingdom | Italy | Germany ) - Football scores

Search Query:

Showing content from https://agda.github.io/agda-stdlib/master/IO.Effectful.html below:

IO.Effectful

IO.Effectful
------------------------------------------------------------------------
-- The Agda standard library
--
-- An effectful view of IO
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --guardedness #-}

module IO.Effectful where

open import Level using (Level; _⊔_)
open import Effect.Functor using (RawFunctor)
open import Effect.Applicative using (RawApplicative)
open import Effect.Monad using (RawMonad)

open import IO.Base

private
  variable
    f : Level

------------------------------------------------------------------------
-- Structure

functor : RawFunctor {f} IO
functor = record { _<$>_ = _<$>_ }

applicative : RawApplicative {f} IO
applicative = record
  { rawFunctor = functor
  ; pure = pure
  ; _<*>_ = _<*>_
  }

monad : RawMonad {f} IO
monad = record
  { rawApplicative = applicative
  ; _>>=_ = _>>=_
  }

RetroSearch is an open source project built by @garambo | Open a GitHub Issue

Search and Browse the WWW like it's 1997 | Search results from DuckDuckGo

HTML: 3.2 | Encoding: UTF-8 | Version: 0.7.4