lean2/tests/lean/run/coe6.lean
Leonardo de Moura 653141135d chore(tests/lean): add missing tests
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-09-04 15:04:57 -07:00

15 lines
339 B
Text

import data.unit
open unit
variable int : Type.{1}
variable nat : Type.{1}
variable izero : int
variable nzero : nat
variable isucc : int → int
variable nsucc : nat → nat
definition f [coercion] (a : unit) : int := izero
definition g [coercion] (a : unit) : nat := nzero
set_option pp.coercion true
check isucc star
check nsucc star