Skip to content

Commit e32b4fc

Browse files
committed
refactor: functoriality of the adjoints, again
1 parent cbf3cc8 commit e32b4fc

File tree

1 file changed

+4
-2
lines changed

1 file changed

+4
-2
lines changed

src/Relation/Unary/Properties.agda

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -245,10 +245,12 @@ module _ {P : Pred A ℓ₁} {Q : Pred B ℓ₂} (f : A → B) where
245245
module _ {P : Pred A ℓ₁} {Q : Pred A ℓ₂} (f : A B) where
246246

247247
map-⟨_⟩⊢_ : P ⊆ Q ⟨ f ⟩⊢ P ⊆ ⟨ f ⟩⊢ Q
248-
map-⟨_⟩⊢_ P⊆Q = ⟨ f ⟩⊢⁺ ⊆-trans {j = Q} P⊆Q (⟨ f ⟩⊢⁻ ⊆-refl {x = ⟨ f ⟩⊢ Q})
248+
map-⟨_⟩⊢_ P⊆Q = ⟨ f ⟩⊢⁺ ⊆-trans {k = f ⊢ ⟨f⟩⊢Q} P⊆Q (⟨ f ⟩⊢⁻ ⊆-refl {x = ⟨f⟩⊢Q})
249+
where ⟨f⟩⊢Q = ⟨ f ⟩⊢ Q
249250

250251
map-[_]⊢_ : P ⊆ Q [ f ]⊢ P ⊆ [ f ]⊢ Q
251-
map-[_]⊢_ P⊆Q = [ f ]⊢⁺ ⊆-trans {j = P} ([ f ]⊢⁻ ⊆-refl {x = [ f ]⊢ P}) P⊆Q
252+
map-[_]⊢_ P⊆Q = [ f ]⊢⁺ ⊆-trans {i = f ⊢ [f]⊢P} ([ f ]⊢⁻ ⊆-refl {x = [f]⊢P}) P⊆Q
253+
where [f]⊢P = [ f ]⊢ P
252254

253255

254256
------------------------------------------------------------------------

0 commit comments

Comments
 (0)