lean2/tests/lean/coe.lean
2014-10-02 17:55:34 -07:00

12 lines
251 B
Text

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
constant f : Functor
check f 0 = 0