Set: pp::colors Set: pp::unicode Assumed: f λ (A B : Type) (a : B), f B a Failed to solve A : Type, a : ?M::0, B : Type ⊢ ?M::0[lift:0:2] ≺ B (line: 4: pos: 42) Type of argument 2 must be convertible to the expected type in the application of f with arguments: B a Assumed: myeq myeq (Π (A : Type), A → A) (λ (A : Type) (a : A), a) (λ (B : Type) (b : B), b) myeq (Π (A : Type), A → A) (λ (A : Type) (a : A), a) (λ (B : Type) (b : B), b) : Bool Assumed: R Assumed: h λ (H : Bool) (f1 g1 : Π A : Type, R A) (G : Π A : Type, myeq (R A) (f1 A) (g1 A)), h f1 : Bool → (Π (f1 g1 : Π A : Type, R A), (Π A : Type, myeq (R A) (f1 A) (g1 A)) → Bool)