4c6b0dc0e5
fixes #466
14 lines
179 B
Text
14 lines
179 B
Text
open eq
|
|
|
|
context
|
|
parameter (A : Type)
|
|
|
|
definition foo (a : A) : a = a := refl a
|
|
|
|
definition bar (a : A) : foo a = refl a :=
|
|
begin
|
|
unfold foo,
|
|
apply rfl
|
|
end
|
|
|
|
end
|