9 lines
99 B
Plaintext
9 lines
99 B
Plaintext
|
import Aesop
|
|||
|
|
|||
|
example : α → α :=
|
|||
|
by aesop
|
|||
|
|
|||
|
theorem eg2 : α → α := by
|
|||
|
intro a
|
|||
|
exact a
|