Skip to content

Commit

Permalink
Applying suggestions
Browse files Browse the repository at this point in the history
  • Loading branch information
viktorcsimma authored and omelkonian committed Mar 1, 2024
1 parent 6959429 commit bb89fd2
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 9 deletions.
8 changes: 2 additions & 6 deletions lib/Haskell/Prim/Applicative.agda
Original file line number Diff line number Diff line change
Expand Up @@ -16,9 +16,7 @@ open import Haskell.Prim.Tuple

-- ** base
record Applicative (f : Set Set) : Set₁ where
infixl 4 _<*>_
infixl 4 _<*_
infixl 4 _*>_
infixl 4 _<*>_ _<*_ _*>_
field
pure : a f a
_<*>_ : f (a b) f a f b
Expand All @@ -28,9 +26,7 @@ record Applicative (f : Set → Set) : Set₁ where
-- ** defaults
record DefaultApplicative (f : Set Set) : Set₁ where
constructor mk
infixl 4 _<*>_
infixl 4 _<*_
infixl 4 _*>_
infixl 4 _<*>_ _<*_ _*>_
field
pure : a f a
_<*>_ : f (a b) f a f b
Expand Down
6 changes: 3 additions & 3 deletions lib/Haskell/Prim/String.agda
Original file line number Diff line number Diff line change
Expand Up @@ -7,10 +7,10 @@ open import Haskell.Prim.Foldable

--------------------------------------------------
-- String
-- This is _not_ the builtin String type of Agda;
-- This is _not_ the builtin String type of Agda
-- which is defined by postulates.
-- fromString can be used to produce Haskell strings
-- from that.
-- `fromString` can be used to convert back
-- to builtin Agda strings.

String = List Char

Expand Down

0 comments on commit bb89fd2

Please sign in to comment.