File tree Expand file tree Collapse file tree 2 files changed +21
-1
lines changed Expand file tree Collapse file tree 2 files changed +21
-1
lines changed Original file line number Diff line number Diff line change @@ -238,6 +238,12 @@ Additions to existing modules
238238 contradiction′ : ¬ A → A → Whatever
239239 ```
240240
241+ * In ` Relation.Unary `
242+ ``` agda
243+ ⟨_⟩⊢_ : (A → B) → Pred A ℓ → Pred B _
244+ [_]⊢_ : (A → B) → Pred A ℓ → Pred B _
245+ ```
246+
241247* In ` System.Random ` :
242248 ``` agda
243249 randomIO : IO Bool
Original file line number Diff line number Diff line change @@ -202,7 +202,7 @@ Decidable P = ∀ x → Dec (P x)
202202-- Operations on sets
203203
204204infix 10 ⋃ ⋂
205- infixr 9 _⊢_
205+ infixr 9 _⊢_ ⟨_⟩⊢_ [_]⊢_
206206infixr 8 _⇒_
207207infixr 7 _∩_
208208infixr 6 _∪_
@@ -266,6 +266,20 @@ P ⊥′ Q = P ∩ Q ⊆′ ∅
266266_⊢_ : (A → B) → Pred B ℓ → Pred A ℓ
267267f ⊢ P = λ x → P (f x)
268268
269+ -- Diamond/Box: for given `f`, these are the left- and right adjoints to `f ⊢_`
270+ -- These are specialization of Diamond/Box in
271+ -- Relation.Unary.Closure.Base.
272+
273+ -- Diamond
274+
275+ ⟨_⟩⊢_ : (A → B) → Pred A ℓ → Pred B _
276+ ⟨ f ⟩⊢ P = λ b → ∃ λ a → f a ≡ b × P a
277+
278+ -- Box
279+
280+ [_]⊢_ : (A → B) → Pred A ℓ → Pred B _
281+ [ f ]⊢ P = λ b → ∀ a → f a ≡ b → P a
282+
269283------------------------------------------------------------------------
270284-- Predicate combinators
271285
You can’t perform that action at this time.
0 commit comments