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 1010
1111module Debug.Trace where
1212
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 (_≡_)
1515
1616-- Postulating the `trace` function and explaining how to compile it
1717
Original file line number Diff line number Diff line change @@ -14,11 +14,9 @@ module Effect.Applicative where
1414open import Data.Bool.Base using (Bool; true; false)
1515open import Data.Product.Base using (_×_; _,_)
1616open import Data.Unit.Polymorphic.Base using (⊤)
17-
1817open import Effect.Choice using (RawChoice)
1918open import Effect.Empty using (RawEmpty)
2019open import Effect.Functor as Fun using (RawFunctor)
21-
2220open import Function.Base using (const; flip; _∘′_)
2321open import Level using (Level; suc; _⊔_)
2422open 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
1313
1414open import Effect.Functor using (RawFunctor)
1515open 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; _⊔_)
1818open import Relation.Binary.PropositionalEquality.Core using (_≡_; refl; cong₂)
1919open import Relation.Binary.PropositionalEquality.Properties
2020 using (module ≡-Reasoning )
Original file line number Diff line number Diff line change @@ -14,8 +14,8 @@ module Effect.Applicative.Predicate where
1414open import Effect.Functor.Predicate
1515open import Data.Product.Base using (_,_)
1616open 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 (_⊆_; _⇒_; _∩_)
1919open import Relation.Unary.PredicateTransformer using (Pt)
2020
2121private
Original file line number Diff line number Diff line change 1010
1111module Effect.Comonad where
1212
13- open import Level
13+ open import Level using (Level; suc)
1414open import Function.Base using (id; _∘′_; flip)
1515
1616private
Original file line number Diff line number Diff line change 88
99module Effect.Empty where
1010
11- open import Level
11+ open import Level using (Level; suc; _⊔_)
1212
1313private
1414 variable
Original file line number Diff line number Diff line change @@ -13,11 +13,8 @@ module Effect.Foldable where
1313open import Algebra.Bundles.Raw using (RawMonoid)
1414open import Algebra.Bundles using (Monoid)
1515import Algebra.Construct.Flip.Op as Op
16-
1716open import Data.List.Base as List using (List; [_]; _++_)
18-
1917open import Effect.Functor as Fun using (RawFunctor)
20-
2118open import Function.Base using (id; flip)
2219open import Function.Endo.Propositional using (∘-id-monoid)
2320open import Level using (Level; Setω)
Original file line number Diff line number Diff line change @@ -12,8 +12,7 @@ module Effect.Functor where
1212
1313open import Data.Unit.Polymorphic.Base using (⊤)
1414open import Function.Base using (const; flip)
15- open import Level
16-
15+ open import Level using (Level; suc; _⊔_)
1716open import Relation.Binary.PropositionalEquality.Core using (_≡_)
1817
1918private
Original file line number Diff line number Diff line change 1111module Effect.Functor.Predicate where
1212
1313open 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 (_⊆_)
1616open import Relation.Unary.PredicateTransformer using (PT)
1717
1818private
Original file line number Diff line number Diff line change @@ -12,10 +12,10 @@ module Effect.Monad where
1212
1313open import Data.Bool.Base using (Bool; true; false; not)
1414open 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)
1919open import Function.Base using (id; flip; _$′_; _∘′_)
2020open import Level using (Level; suc; _⊔_)
2121
You can’t perform that action at this time.
0 commit comments