lean2/tests/lean/cases_tac.lean.expected.out
Sebastian Ullrich 77c20e99ff feat(library/tactic/inversion_tactic): consistent orientation of generated equalities
Generated equalities in proof irrelevant environments were inverted
compared with the documentation and the proof relevant case, which
resulted in newly generated local vars replacing equivalent old ones
instead of the other way around.
2015-05-14 23:32:54 +02:00

14 lines
220 B
Text

cases_tac.lean:7:2: proof state
A : Type,
B : A → Type,
a : A,
Hb : B a
⊢ A
cases_tac.lean:17:2: proof state
A : Type,
B : A → Type,
f : A → A,
a : A,
Hc : a = a,
Hb : foo₂.mk (f a) a = foo₂.mk (f a) a
⊢ A