lean2/tests/lean/unifier_bug.lean
Leonardo de Moura ea739100b3 fix(library/unifier): broken optimization in the unifier
See new comments and tests for details.
2014-10-28 16:09:41 -07:00

7 lines
200 B
Text

import logic
theorem test {A B : Type} {a : A} {b : B} (H : a == b) :
eq.rec_on (heq.type_eq H) a = b
:=
-- Remark the error message should not occur in the token theorem
heq.rec_on H rfl