lean2/tests/lean/run/ctx.lean

23 lines
363 B
Text
Raw Normal View History

import data.nat
2014-09-09 23:21:30 +00:00
open nat inhabited
constant N : Type.{1}
constant a : N
2014-09-09 23:21:30 +00:00
section s1
set_option pp.implicit true
definition f (a b : nat) := a
theorem nat_inhabited [instance] : inhabited nat :=
inhabited.mk zero
definition to_N [coercion] (n : nat) : N := a
infixl `$$`:65 := f
end s1
theorem tst : inhabited nat
constants n m : nat
2014-09-09 23:21:30 +00:00
check n = a