2014-10-05 17:50:13 +00:00
|
|
|
import data.nat logic.inhabited
|
2014-09-09 23:21:30 +00:00
|
|
|
open nat inhabited
|
|
|
|
|
2014-10-02 23:20:52 +00:00
|
|
|
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
|
2014-10-02 23:20:52 +00:00
|
|
|
constants n m : nat
|
2014-09-09 23:21:30 +00:00
|
|
|
check n = a
|