agda-gset/Preliminaries.agda

5 lines
220 B
Agda
Raw Normal View History

2024-05-05 14:43:35 +02:00
module Preliminaries where
open import Relation.Binary.PropositionalEquality as using (_≡_) public
postulate
FunExt : {} {X Y : Set } {f g : X Y} ( (x : X) f x g x) f g