lean2/tests/lean/run/nat_coe.lean
Leonardo de Moura 08ae17650b feat(frontends/lean): try overloaded notation and declarations in the order they were defined
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-08-18 18:58:50 -07:00

26 lines
414 B
Text

import logic
variable nat : Type.{1}
variable int : Type.{1}
variable nat_add : nat → nat → nat
infixl `+`:65 := nat_add
variable int_add : int → int → int
infixl `+`:65 := int_add
variable of_nat : nat → int
coercion of_nat
variables a b : nat
variables i j : int
abbreviation c1 := a + b
theorem T1 : c1 = nat_add a b :=
refl _
abbreviation c2 := i + j
theorem T2 : c2 = int_add i j :=
refl _