We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
2 parents a390fc0 + 38f22ec commit 7ad3526Copy full SHA for 7ad3526
src/Relation/Unary.agda
@@ -202,7 +202,7 @@ Decidable P = ∀ x → Dec (P x)
202
-- Operations on sets
203
204
infix 10 ⋃ ⋂
205
-infixr 9 _⊢_
+infixr 9 _⊢_ ⟨_⟩⊢_ [_]⊢_
206
infixr 8 _⇒_
207
infixr 7 _∩_
208
infixr 6 _∪_
@@ -277,9 +277,13 @@ f ⊢ P = λ x → P (f x)
277
-- In some settings, the left adjoint is called 'image' or 'pushforward',
278
-- but the right adjoint doesn't seem to have a non-symbolic name.
279
280
+-- Diamond
281
+
282
⟨_⟩⊢_ : (A → B) → Pred A ℓ → Pred B _
283
⟨ f ⟩⊢ P = λ y → ∃ λ x → f x ≡ y × P x
284
285
+-- Box
286
287
[_]⊢_ : (A → B) → Pred A ℓ → Pred B _
288
[ f ]⊢ P = λ y → ∀ {x} → f x ≡ y → P x
289
0 commit comments