@@ -261,21 +261,26 @@ P ⊥ Q = P ∩ Q ⊆ ∅
261261_⊥′_ : Pred A ℓ₁ → Pred A ℓ₂ → Set _
262262P ⊥′ Q = P ∩ Q ⊆′ ∅
263263
264- -- Update/functorial change-of-base
265-
266- -- The notation captures the Martin-Löf tradition of only mentioning
267- -- updates to the ambient context when describing a context-indexed
268- -- family P e.g. (_, σ) ⊢ Tm τ is
264+ -- Update/preimage/inverse image/functorial change-of-base
265+ --
266+ -- The notation, which elsewhere might be rendered
267+ -- * `f⁻¹ P`, for preimage/inverse image
268+ -- * `f* P`, for change-of-base/pullback along `f`
269+ -- captures the Martin-Löf tradition of only mentioning updates to
270+ -- the ambient context when describing a context-indexed family P:
271+ -- e.g. (_, σ) ⊢ Tm τ is
269272-- "a term of type τ in the ambient context extended with a fresh σ".
270273
271274_⊢_ : (A → B) → Pred B ℓ → Pred A ℓ
272275f ⊢ P = λ x → P (f x)
273276
274277-- Change-of-base has left- and right- adjoints (Lawvere).
278+ --
275279-- We borrow the 'diamond'/'box' notation from modal logic, cf.
276280-- `Relation.Unary.Closure.Base`, rather than Lawvere's ∃f, ∀f.
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.
281+ -- In some settings (eg statistics/probability), the left adjoint
282+ -- is called 'image' or 'pushforward', but the right adjoint
283+ -- doesn't seem to have a non-symbolic name.
279284
280285-- Diamond
281286
0 commit comments