erase function argument of cong

This commit is contained in:
Alex Gryzlov 2020-05-24 05:16:52 +02:00
parent cf7de2201f
commit 723f690f7e

View File

@ -117,7 +117,7 @@ public export
||| Equality is a congruence.
public export
cong : (f : t -> u) -> (1 p : a = b) -> f a = f b
cong : (0 f : t -> u) -> (1 p : a = b) -> f a = f b
cong f Refl = Refl
||| A canonical proof that some type is empty.