We have the pointwise PropositionalEquality definition _≗_ (moved in #2335 )
_≗_ {A = A} {B = B} f g = ∀ x → f x ≡ g xand the Function definition _≈_ (since #2240 and its antecedent issues back to #1467 )
_≈_ : (f g : Func From To) → Set (a₁ ⊔ b₂)
f ≈ g = {x : From.Carrier} → f ⟨$⟩ x To.≈ g ⟨$⟩ xand... we are (once again!) inconsistent as to implicit/explicit quantification.
@JacquesCarette has argued for the implicit version; @Taneb 's recent topic thread on Zulip 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.