79d0347721
Remark: the intros tactic has been added in a different commit: 7d0100a340
11 lines
258 B
Text
11 lines
258 B
Text
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
|