lean2/tests/lean/run/rat_rfl.lean
Leonardo de Moura 2d22bb8ea2 feat(frontends/lean/builtin_cmds): do not unfold proofs in the eval command
In the future, we should probably add an option for unfolding proofs.
2015-05-20 19:14:57 -07:00

7 lines
113 B
Text

import data.rat
open rat
attribute rat.of_int [coercion]
example : 1 + 2⁻¹ + 3 = 3 + 2⁻¹ + 1⁻¹ :=
rfl