-
Notifications
You must be signed in to change notification settings - Fork 381
Open
Labels
hidden argumentsInsertion of hidden arguments and implicit lambdasInsertion of hidden arguments and implicit lambdas
Description
This kind of thing has been hitting me repeatedly recently (eg in agda/agda-stdlib#2782): bad interaction between using a lemma from stdlib
, with 'obvious' instantiation, but implicit/explicit argument checking seems to trigger an error. Very poor UX! Message is incomprehensible, and reason for triggering error also incomprehensible. If there's a fix that makes the stdlib
UX smoother for users, please advise!
module MWE where
open import Relation.Nullary.Negation.Core using (¬_; contradiction)
postulate
A : Set
P : A → Set
∀P : ∀ {a} → P a
¬∀P : ¬ (∀ {a} → P a)
test = contradiction ∀P ¬∀P
Tested with:
- v2.8.0
- current
master
ofstdlib
, but any v2.x version should reproduce
Metadata
Metadata
Assignees
Labels
hidden argumentsInsertion of hidden arguments and implicit lambdasInsertion of hidden arguments and implicit lambdas