File tree Expand file tree Collapse file tree 1 file changed +13
-1
lines changed
Mathlib/Combinatorics/SimpleGraph Expand file tree Collapse file tree 1 file changed +13
-1
lines changed Original file line number Diff line number Diff line change @@ -1311,10 +1311,22 @@ theorem map_injective_of_injective {f : G →g G'} (hinj : Function.Injective f)
13111311 apply ih
13121312 simpa using h.2
13131313
1314+ section mapLe
1315+
1316+ variable {G G' : SimpleGraph V} (h : G ≤ G') {u v : V} (p : G.Walk u v)
1317+
13141318/-- The specialization of `SimpleGraph.Walk.map` for mapping walks to supergraphs. -/
1315- abbrev mapLe {G G' : SimpleGraph V} (h : G ≤ G') {u v : V} (p : G.Walk u v) : G'.Walk u v :=
1319+ abbrev mapLe : G'.Walk u v :=
13161320 p.map (.ofLE h)
13171321
1322+ lemma support_mapLe_eq_support : (p.mapLe h).support = p.support := by simp
1323+
1324+ lemma edges_mapLe_eq_edges : (p.mapLe h).edges = p.edges := by simp
1325+
1326+ lemma edgeSet_mapLe_eq_edgeSet : (p.mapLe h).edgeSet = p.edgeSet := by simp
1327+
1328+ end mapLe
1329+
13181330/-! ### Transferring between graphs -/
13191331
13201332/-- The walk `p` transferred to lie in `H`, given that `H` contains its edges. -/
You can’t perform that action at this time.
0 commit comments