Set: pp::colors Set: pp::unicode Imported 'cast' Set: pp::colors λ (A A' : TypeM) (B : A → TypeM) (B' : A' → TypeM) (f : ∀ x : A, B x) (g : ∀ x : A', B' x) (a : A) (b : A') (H2 : f == g) (H3 : a == b), hcongr H2 H3 : ∀ (A A' : TypeM) (B : A → TypeM) (B' : A' → TypeM) (f : ∀ x : A, B x) (g : ∀ x : A', B' x) (a : A) (b : A'), f == g → a == b → f a == g b