2014-09-20 16:56:46 +00:00
|
|
|
import logic
|
|
|
|
|
|
|
|
set_option pp.notation false
|
|
|
|
|
|
|
|
inductive Functor :=
|
|
|
|
mk : (Π (A B : Type), A → B) → Functor
|
|
|
|
|
|
|
|
definition Functor.to_fun [coercion] (f : Functor) {A B : Type} : A → B :=
|
|
|
|
Functor.rec (λ f, f) f A B
|
|
|
|
|
2014-10-02 23:20:52 +00:00
|
|
|
constant f : Functor
|
2014-09-20 16:56:46 +00:00
|
|
|
check f 0 = 0
|