lean2/tests/lean/run/rat_rfl.lean

8 lines
113 B
Text
Raw Normal View History

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