Skip to content

Commit

Permalink
chore: use explicit max func in spine_map_vertex
Browse files Browse the repository at this point in the history
  • Loading branch information
gio256 committed Jan 18, 2025
1 parent 48bb968 commit 7a07689
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicTopology/SimplicialSet/Path.lean
Original file line number Diff line number Diff line change
Expand Up @@ -205,7 +205,7 @@ lemma spine_map_vertex {n : ℕ} (Δ : X _[n]) {m : ℕ} (φ : [m] ⟶ [n])
(i : Fin (m + 1)) :
(spine X m (X.map φ.op Δ)).vertex i =
(spine X n Δ).vertex (φ.toOrderHom i) :=
truncation ((m ⊔ n) + 1) |>.obj X
truncation (max m n + 1) |>.obj X
|>.spine_map_vertex n (by leq) Δ m (by leq) φ i

/-- The spine of the unique non-degenerate `n`-simplex in `Δ[n]`. -/
Expand Down

0 comments on commit 7a07689

Please sign in to comment.