118189eaac
This commit fixes the bug reported in the lean discussion list: https://groups.google.com/forum/#!topic/lean-discuss/oyzgIqdMyNc
4 lines
127 B
Text
4 lines
127 B
Text
definition s : Type := sorry
|
|
|
|
example (A : Type) (s : A) : A := by exact s
|
|
example (A : Type) : A → A := by intro s; exact s
|