File tree 5 files changed +5
-5
lines changed
5 files changed +5
-5
lines changed Original file line number Diff line number Diff line change @@ -49,7 +49,7 @@ monad = record
49
49
}
50
50
51
51
-- The monad instance also requires some mucking about with universe levels.
52
- monadT : RawMonadT (_∘′ Productₗ)
52
+ monadT : ∀ {ℓ} → RawMonadT {g₁ = ℓ} (_∘′ Productₗ)
53
53
monadT M = record
54
54
{ lift = (ε ,_) <$>_
55
55
; rawMonad = mkRawMonad _
Original file line number Diff line number Diff line change @@ -48,7 +48,7 @@ monad = record
48
48
; _>>=_ = uncurry λ a w₁ f → map₂ (w₁ ∙_) (f a)
49
49
}
50
50
51
- monadT : RawMonadT (_∘′ Productᵣ)
51
+ monadT : ∀ {ℓ} → RawMonadT {g₁ = ℓ} (_∘′ Productᵣ)
52
52
monadT M = record
53
53
{ lift = (_, ε) <$>_
54
54
; rawMonad = mkRawMonad _
Original file line number Diff line number Diff line change @@ -77,7 +77,7 @@ module _ where
77
77
78
78
-- Smart constructor
79
79
mkRawApplicative :
80
- (F : Set f → Set f ) →
80
+ (F : Set f → Set g ) →
81
81
(pure : ∀ {A} → A → F A) →
82
82
(app : ∀ {A B} → F (A → B) → F A → F B) →
83
83
RawApplicative F
Original file line number Diff line number Diff line change @@ -74,7 +74,7 @@ module _ where
74
74
open RawApplicative
75
75
76
76
mkRawMonad :
77
- (F : Set f → Set f ) →
77
+ (F : Set f → Set g ) →
78
78
(pure : ∀ {A} → A → F A) →
79
79
(bind : ∀ {A B} → F A → (A → F B) → F B) →
80
80
RawMonad F
Original file line number Diff line number Diff line change @@ -116,7 +116,7 @@ module _ where
116
116
module _ where
117
117
118
118
private
119
- anyApplicative : RawApplicative (λ _ → Bool)
119
+ anyApplicative : ∀ {ℓ} → RawApplicative {ℓ} (λ _ → Bool)
120
120
anyApplicative = mkRawApplicative _ (λ _ → false) _∨_
121
121
122
122
open Traverse anyApplicative
You can’t perform that action at this time.
0 commit comments