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

20 lines
472 B
Text

import data.fin
open nat
namespace fin
definition z_cases_on2 (C : fin zero → Type) (p : fin zero) : C p :=
by cases p
definition nz_cases_on2 {C : Π n, fin (succ n) → Type}
(H₁ : Π n, C n (fz n))
(H₂ : Π n (f : fin n), C n (fs f))
{n : nat}
(f : fin (succ n)) : C n f :=
begin
cases f,
apply (H₁ n),
apply (H₂ n a)
end
end fin