lean2/tests/lean/cases_tac.lean
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

19 lines
412 B
Text

inductive foo {A : Type} : A → Type :=
mk : Π a : A, foo a
example (A : Type) (B : A → Type) (a : A) (H : foo a) (Hb : B a) : A :=
begin
cases H,
state,
assumption
end
inductive foo₂ {A : Type} : A → A → Type :=
mk : Π a b : A, foo₂ a b
example (A : Type) (B : A → Type) (f : A → A) (a : A) (H : foo₂ (f a) a) (Hb : H = H) (Hc : a = a) : A :=
begin
cases H,
state,
exact a
end