We have [the pointwise `PropositionalEquality` definition `_≗_`](https://github.com/agda/agda-stdlib/blob/c719430e5f27a2df47a18df8781cb5824ba5b601/src/Relation/Binary/PropositionalEquality/Core.agda#L35-L42) (moved in #2335 ) ```agda _≗_ {A = A} {B = B} f g = ∀ x → f x ≡ g x ``` and [the `Function` definition `_≈_`](https://github.com/agda/agda-stdlib/blob/c719430e5f27a2df47a18df8781cb5824ba5b601/src/Function/Relation/Binary/Setoid/Equality.agda#L25-L27) (since #2240 and its antecedent issues back to #1467 ) ```agda _≈_ : (f g : Func From To) → Set (a₁ ⊔ b₂) f ≈ g = {x : From.Carrier} → f ⟨$⟩ x To.≈ g ⟨$⟩ x ``` and... we are (once again!) inconsistent as to implicit/explicit quantification. @JacquesCarette has argued for the implicit version; @Taneb 's recent [topic thread on Zulip](https://agda.zulipchat.com/#narrow/stream/263194-categories/topic/Should.20Sets.20use.20.E2.89.97.3F) suggests that this is not always the right choice. Maybe there's room for both, but it doesn't feel quite right to me... or else, the distinction should be documented.