mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-11 02:01:36 +03:00
erase function argument of cong
This commit is contained in:
parent
cf7de2201f
commit
723f690f7e
@ -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.
|
||||
|
Loading…
Reference in New Issue
Block a user