lean2/tests/lean/691.lean
2015-06-28 11:28:05 -07:00

13 lines
203 B
Text

theorem foo : Type₁ := unit
example : foo = unit :=
by unfold foo
example : foo = unit :=
by unfold [foo]
example : foo = unit :=
by rewrite [↑foo]
example : foo = unit :=
by rewrite [↑[foo] ]