lean2/tests/lean/run/calc_bug.lean
Leonardo de Moura bc65aeb5e1 fix(frontends/lean/calc): add expected type for single-step calc expressions, fixes #357
This is not an issue for calc expressions containing multiple steps,
since the transitivity step will "force" the expected type for the proofs.
2014-11-29 15:35:09 -08:00

4 lines
60 B
Text

import logic
definition foo (a : Type) :=
calc a = a : rfl