14 lines
203 B
Text
14 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] ]
|