Skip to content

Commit 7ad3526

Browse files
authored
Merge branch 'master' into unary-adjoints
2 parents a390fc0 + 38f22ec commit 7ad3526

File tree

1 file changed

+5
-1
lines changed

1 file changed

+5
-1
lines changed

src/Relation/Unary.agda

Lines changed: 5 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -202,7 +202,7 @@ Decidable P = ∀ x → Dec (P x)
202202
-- Operations on sets
203203

204204
infix 10 ⋃ ⋂
205-
infixr 9 _⊢_
205+
infixr 9 _⊢_ ⟨_⟩⊢_ [_]⊢_
206206
infixr 8 _⇒_
207207
infixr 7 _∩_
208208
infixr 6 _∪_
@@ -277,9 +277,13 @@ f ⊢ P = λ x → P (f x)
277277
-- In some settings, the left adjoint is called 'image' or 'pushforward',
278278
-- but the right adjoint doesn't seem to have a non-symbolic name.
279279

280+
-- Diamond
281+
280282
⟨_⟩⊢_ : (A B) Pred A ℓ Pred B _
281283
⟨ f ⟩⊢ P = λ y λ x f x ≡ y × P x
282284

285+
-- Box
286+
283287
[_]⊢_ : (A B) Pred A ℓ Pred B _
284288
[ f ]⊢ P = λ y {x} f x ≡ y P x
285289

0 commit comments

Comments
 (0)