Skip to content

Regression related to fix of #3027 #4408

Closed
@nad

Description

@nad

The following code is accepted by Agda 2.6.0.1, but rejected by a recent development version:

comp :
  (A : Set)
  (B : A  Set)
  (C : (x : A)  B x  Set) 
  ((x : A) (y : B x)  C x y) 
  (g : (x : A)  B x) 
  ((x : A)  C x (g x))
comp _ _ _ f g x = f x (g x)

data Unit : Set where
  unit : Unit

P : Unit  Set
P unit = Unit

Q : Unit  Set  Set
Q unit = λ _  Unit

f : (x : Unit)  P x  P x
f unit x = x

g :
  (A : Set) 
  ((x : Unit)  Q x A  P x) 
  ((x : Unit)  Q x A  P x)
g A h x = comp _ _ _ (λ _  f _) (h _)

Bisection points towards 3c6482b ("[ fix #3027 ] block bound variable on right side of constraint (#4392)"). @vlopezj, you might want to take a look at this.

Metadata

Metadata

Assignees

Labels

constraintsConstraints (postponed type checking problems, postponed unification problems, instance constraints)metaMetavariables, insertion of implicit arguments, etcregression on masterUnreleased regression in development version (Change to "regression in ..." should it be released!)

Type

No type

Projects

No projects

Milestone

Relationships

None yet

Development

No branches or pull requests

Issue actions