lean2/tests/lean/coercion1.lean
Leonardo de Moura 42be7a4989 Add coercion declarations
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-09-01 18:11:28 -07:00

16 lines
299 B
Text

Set pp::colors false
Variable T : Type
Variable R : Type
Variable f : T -> R
Coercion f
Show Environment 2
Variable g : T -> R
Coercion g
Variable h : Pi (x : Type), x
Coercion h
Definition T2 : Type := T
Definition R2 : Type := R
Variable f2 : T2 -> R2
Coercion f2
Variable id : T -> T
Coercion id