Rewriting arrows and paths along vertex equalities #
This files defines Hom.cast
and Path.cast
(and associated lemmas) in order to allow
rewriting arrows and paths along equalities of their endpoints.
Rewriting arrows along equalities of vertices #
def
Quiver.Hom.cast
{U : Type u_1}
[Quiver U]
{u v u' v' : U}
(hu : u = u')
(hv : v = v')
(e : u ⟶ v)
:
u' ⟶ v'
Change the endpoints of an arrow using equalities.
Equations
- Quiver.Hom.cast hu hv e = hu ▸ hv ▸ e
Instances For
theorem
Quiver.Hom.cast_eq_cast
{U : Type u_1}
[Quiver U]
{u v u' v' : U}
(hu : u = u')
(hv : v = v')
(e : u ⟶ v)
:
cast hu hv e = _root_.cast ⋯ e
Rewriting paths along equalities of vertices #
def
Quiver.Path.cast
{U : Type u_1}
[Quiver U]
{u v u' v' : U}
(hu : u = u')
(hv : v = v')
(p : Path u v)
:
Path u' v'
Change the endpoints of a path using equalities.
Equations
- Quiver.Path.cast hu hv p = hu ▸ hv ▸ p
Instances For
theorem
Quiver.Path.cast_eq_cast
{U : Type u_1}
[Quiver U]
{u v u' v' : U}
(hu : u = u')
(hv : v = v')
(p : Path u v)
:
cast hu hv p = _root_.cast ⋯ p