Skip to content

Commit cbf3cc8

Browse files
committed
refactor: functoriality of the adjoints
1 parent 8bf7322 commit cbf3cc8

File tree

1 file changed

+8
-8
lines changed

1 file changed

+8
-8
lines changed

src/Relation/Unary/Properties.agda

Lines changed: 8 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -228,14 +228,6 @@ module _ {P : Pred B ℓ₁} {Q : Pred B ℓ₂} where
228228
_map-⊢_ : (f : A B) P ⊆ Q f ⊢ P ⊆ f ⊢ Q
229229
f map-⊢ P⊆Q = P⊆Q
230230

231-
module _ {P : Pred A ℓ₁} {Q : Pred A ℓ₂} (f : A B) where
232-
233-
map-⟨_⟩⊢_ : P ⊆ Q ⟨ f ⟩⊢ P ⊆ ⟨ f ⟩⊢ Q
234-
map-⟨_⟩⊢_ P⊆Q (_ , refl , Px) = (_ , refl , P⊆Q Px)
235-
236-
map-[_]⊢_ : P ⊆ Q [ f ]⊢ P ⊆ [ f ]⊢ Q
237-
map-[_]⊢_ P⊆Q Px refl = P⊆Q (Px refl)
238-
239231
module _ {P : Pred A ℓ₁} {Q : Pred B ℓ₂} (f : A B) where
240232

241233
⟨_⟩⊢⁻_ : ⟨ f ⟩⊢ P ⊆ Q P ⊆ f ⊢ Q
@@ -250,6 +242,14 @@ module _ {P : Pred A ℓ₁} {Q : Pred B ℓ₂} (f : A → B) where
250242
[_]⊢⁺_ : f ⊢ Q ⊆ P Q ⊆ [ f ]⊢ P
251243
[_]⊢⁺_ f⊢Q⊆P Qfx refl = f⊢Q⊆P Qfx
252244

245+
module _ {P : Pred A ℓ₁} {Q : Pred A ℓ₂} (f : A B) where
246+
247+
map-⟨_⟩⊢_ : P ⊆ Q ⟨ f ⟩⊢ P ⊆ ⟨ f ⟩⊢ Q
248+
map-⟨_⟩⊢_ P⊆Q = ⟨ f ⟩⊢⁺ ⊆-trans {j = Q} P⊆Q (⟨ f ⟩⊢⁻ ⊆-refl {x = ⟨ f ⟩⊢ Q})
249+
250+
map-[_]⊢_ : P ⊆ Q [ f ]⊢ P ⊆ [ f ]⊢ Q
251+
map-[_]⊢_ P⊆Q = [ f ]⊢⁺ ⊆-trans {j = P} ([ f ]⊢⁻ ⊆-refl {x = [ f ]⊢ P}) P⊆Q
252+
253253

254254
------------------------------------------------------------------------
255255
-- Decidability properties

0 commit comments

Comments
 (0)