lean2/tests/lean/run/get_tac1.lean

12 lines
258 B
Text
Raw Normal View History

import hott.path tools.tactic
open path
definition concat_pV_p {A : Type} {x y z : A} (p : x ≈ z) (q : y ≈ z) : (p ⬝ q⁻¹) ⬝ q ≈ p :=
begin
generalize p,
apply (path.induction_on q),
intro p,
apply (path.induction_on p),
apply idp
end