lean2/tests/lean/coercion1.lean

16 lines
278 B
Text
Raw Normal View History

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