File tree Expand file tree Collapse file tree 17 files changed +30
-36
lines changed Expand file tree Collapse file tree 17 files changed +30
-36
lines changed Original file line number Diff line number Diff line change 10
10
11
11
module Debug.Trace where
12
12
13
- open import Agda.Builtin.String
14
- open import Agda.Builtin.Equality
13
+ open import Agda.Builtin.String using (String)
14
+ open import Agda.Builtin.Equality using (_≡_)
15
15
16
16
-- Postulating the `trace` function and explaining how to compile it
17
17
Original file line number Diff line number Diff line change @@ -14,11 +14,9 @@ module Effect.Applicative where
14
14
open import Data.Bool.Base using (Bool; true; false)
15
15
open import Data.Product.Base using (_×_; _,_)
16
16
open import Data.Unit.Polymorphic.Base using (⊤)
17
-
18
17
open import Effect.Choice using (RawChoice)
19
18
open import Effect.Empty using (RawEmpty)
20
19
open import Effect.Functor as Fun using (RawFunctor)
21
-
22
20
open import Function.Base using (const; flip; _∘′_)
23
21
open import Level using (Level; suc; _⊔_)
24
22
open import Relation.Binary.PropositionalEquality.Core using (_≡_)
Original file line number Diff line number Diff line change @@ -13,8 +13,8 @@ module Effect.Applicative.Indexed where
13
13
14
14
open import Effect.Functor using (RawFunctor)
15
15
open import Data.Product.Base using (_×_; _,_)
16
- open import Function.Base
17
- open import Level
16
+ open import Function.Base using (const; constᵣ)
17
+ open import Level using (Level; suc; _⊔_)
18
18
open import Relation.Binary.PropositionalEquality.Core using (_≡_; refl; cong₂)
19
19
open import Relation.Binary.PropositionalEquality.Properties
20
20
using (module ≡-Reasoning )
Original file line number Diff line number Diff line change @@ -14,8 +14,8 @@ module Effect.Applicative.Predicate where
14
14
open import Effect.Functor.Predicate
15
15
open import Data.Product.Base using (_,_)
16
16
open import Function.Base using (const; constᵣ)
17
- open import Level
18
- open import Relation.Unary
17
+ open import Level using (Level; suc; _⊔_)
18
+ open import Relation.Unary using (_⊆_; _⇒_; _∩_)
19
19
open import Relation.Unary.PredicateTransformer using (Pt)
20
20
21
21
private
Original file line number Diff line number Diff line change 10
10
11
11
module Effect.Comonad where
12
12
13
- open import Level
13
+ open import Level using (Level; suc)
14
14
open import Function.Base using (id; _∘′_; flip)
15
15
16
16
private
Original file line number Diff line number Diff line change 8
8
9
9
module Effect.Empty where
10
10
11
- open import Level
11
+ open import Level using (Level; suc; _⊔_)
12
12
13
13
private
14
14
variable
Original file line number Diff line number Diff line change @@ -13,11 +13,8 @@ module Effect.Foldable where
13
13
open import Algebra.Bundles.Raw using (RawMonoid)
14
14
open import Algebra.Bundles using (Monoid)
15
15
import Algebra.Construct.Flip.Op as Op
16
-
17
16
open import Data.List.Base as List using (List; [_]; _++_)
18
-
19
17
open import Effect.Functor as Fun using (RawFunctor)
20
-
21
18
open import Function.Base using (id; flip)
22
19
open import Function.Endo.Propositional using (∘-id-monoid)
23
20
open import Level using (Level; Setω)
Original file line number Diff line number Diff line change @@ -12,8 +12,7 @@ module Effect.Functor where
12
12
13
13
open import Data.Unit.Polymorphic.Base using (⊤)
14
14
open import Function.Base using (const; flip)
15
- open import Level
16
-
15
+ open import Level using (Level; suc; _⊔_)
17
16
open import Relation.Binary.PropositionalEquality.Core using (_≡_)
18
17
19
18
private
Original file line number Diff line number Diff line change 11
11
module Effect.Functor.Predicate where
12
12
13
13
open import Function.Base using (const)
14
- open import Level
15
- open import Relation.Unary
14
+ open import Level using (Level; suc; _⊔_)
15
+ open import Relation.Unary using (_⊆_)
16
16
open import Relation.Unary.PredicateTransformer using (PT)
17
17
18
18
private
Original file line number Diff line number Diff line change @@ -12,10 +12,10 @@ module Effect.Monad where
12
12
13
13
open import Data.Bool.Base using (Bool; true; false; not)
14
14
open import Data.Unit.Polymorphic.Base using (⊤)
15
-
16
- open import Effect.Choice
17
- open import Effect.Empty
18
- open import Effect.Applicative
15
+ open import Effect.Choice using (RawChoice)
16
+ open import Effect.Empty using (RawEmpty)
17
+ open import Effect.Applicative as App
18
+ using (RawApplicative; RawApplicativeZero; mkRawApplicative; RawAlternative)
19
19
open import Function.Base using (id; flip; _$′_; _∘′_)
20
20
open import Level using (Level; suc; _⊔_)
21
21
Original file line number Diff line number Diff line change 11
11
module Effect.Monad.Indexed where
12
12
13
13
open import Effect.Applicative.Indexed
14
- open import Function.Base
15
- open import Level
14
+ using (IFun; RawIApplicative; RawIApplicativeZero; RawIAlternative)
15
+ open import Function.Base using (id; _∘_)
16
+ open import Level using (Level; _⊔_; suc)
16
17
17
18
private
18
19
variable
Original file line number Diff line number Diff line change 8
8
9
9
module Effect.Monad.Partiality.All where
10
10
11
- open import Effect.Monad
11
+ open import Effect.Monad using (RawMonad)
12
12
open import Effect.Monad.Partiality as Partiality using (_⊥; ⇒≈)
13
- open import Codata.Musical.Notation
13
+ open import Codata.Musical.Notation using (♭; ∞; ♯_)
14
14
open import Function.Base using (flip; _∘_)
15
- open import Level
15
+ open import Level using (Level; _⊔_; suc)
16
16
open import Relation.Binary.Definitions using (_Respects_)
17
17
open import Relation.Binary.Structures using (IsEquivalence)
18
18
open import Relation.Binary.PropositionalEquality.Core as ≡ using (_≡_)
Original file line number Diff line number Diff line change @@ -14,8 +14,8 @@ open import Function.Base using (const; flip; _∘_)
14
14
open import Function.Identity.Effectful as Id using (Identity)
15
15
open import Effect.Applicative.Indexed
16
16
using (IFun; RawIApplicative; RawIApplicativeZero; RawIAlternative)
17
- open import Effect.Monad.Indexed using (RawIMonad; RawIMonadZero;
18
- RawIMonadPlus)
17
+ open import Effect.Monad.Indexed
18
+ using (RawIMonad; RawIMonadZero; RawIMonadPlus)
19
19
20
20
private
21
21
variable
Original file line number Diff line number Diff line change @@ -12,8 +12,8 @@ open import Effect.Applicative.Indexed
12
12
using (IFun; RawIApplicative; RawIApplicativeZero; RawIAlternative)
13
13
open import Effect.Monad using (RawMonad; RawMonadZero; RawMonadPlus)
14
14
open import Function.Identity.Effectful as Id using (Identity)
15
- open import Effect.Monad.Indexed using (RawIMonad; RawIMonadZero;
16
- RawIMonadPlus)
15
+ open import Effect.Monad.Indexed
16
+ using (RawIMonad; RawIMonadZero; RawIMonadPlus)
17
17
open import Data.Product.Base using (_×_; _,_; uncurry)
18
18
open import Data.Unit.Polymorphic using (⊤)
19
19
open import Function.Base using (const; _∘_)
Original file line number Diff line number Diff line change @@ -11,11 +11,10 @@ module Effect.Monad.State.Transformer.Base where
11
11
12
12
open import Data.Product.Base using (_×_; proj₁; proj₂)
13
13
open import Data.Unit.Polymorphic.Base using (⊤)
14
+ open import Effect.Functor using (RawFunctor)
14
15
open import Function.Base using (_∘′_; const; id)
15
16
open import Level using (Level; suc; _⊔_)
16
17
17
- open import Effect.Functor
18
-
19
18
private
20
19
variable
21
20
f s : Level
Original file line number Diff line number Diff line change @@ -12,10 +12,11 @@ module Effect.Monad.Writer.Indexed (a : Level) where
12
12
13
13
open import Algebra using (RawMonoid)
14
14
open import Data.Product.Base using (_×_; _,_; map₁)
15
- open import Data.Unit.Polymorphic
15
+ open import Data.Unit.Polymorphic using (⊤; tt)
16
16
open import Effect.Applicative.Indexed
17
- open import Effect.Monad
17
+ using (IFun; RawIApplicative; RawIApplicativeZero; RawIAlternative)
18
18
open import Effect.Monad.Indexed
19
+ using (RawIMonad; RawIMonadZero; RawIMonadPlus)
19
20
open import Function.Base using (_∘′_)
20
21
open import Function.Identity.Effectful as Id using (Identity)
21
22
Original file line number Diff line number Diff line change @@ -11,11 +11,10 @@ module Effect.Monad.Writer.Transformer.Base where
11
11
open import Algebra using (RawMonoid)
12
12
open import Data.Product.Base using (_×_; _,_; proj₁; proj₂)
13
13
open import Data.Unit.Polymorphic using (⊤; tt)
14
+ open import Effect.Functor using (RawFunctor)
14
15
open import Function.Base using (id; _∘′_)
15
16
open import Level using (Level; suc; _⊔_)
16
17
17
- open import Effect.Functor using (RawFunctor)
18
-
19
18
private
20
19
variable
21
20
w f g : Level
You can’t perform that action at this time.
0 commit comments