Skip to content

Conversation

@kim-em
Copy link
Contributor

@kim-em kim-em commented Jan 29, 2026

This PR adds Path.subpathOn, which extracts a subpath from a path γ on an interval [a, b] ⊆ [0, 1] by reparametrizing via the affine map t ↦ a + t(b - a).

Main results

  • Path.subpathOn: definition of the restricted path
  • Path.subpathOn_trans: composing subpaths is homotopic to the combined subpath
  • Path.subpathOn_self: the trivial subpath [a,a] is homotopic to the constant path
  • Path.subpathOn_zero_one: the full subpath [0,1] is homotopic to the original path
  • Quotient-level versions of these theorems

This material is split out from #31576 to allow independent review. PR #31576 will depend on this PR once merged.

🤖 Prepared with Claude Code

…subintervals

This PR adds `Path.subpathOn`, which extracts a subpath from a path γ
on an interval [a, b] ⊆ [0, 1] by reparametrizing via the affine map
t ↦ a + t(b - a).

Main results:
- `Path.subpathOn`: definition of the restricted path
- `Path.subpathOn_trans`: composing subpaths is homotopic to the combined subpath
- `Path.subpathOn_self`: the trivial subpath [a,a] is homotopic to the constant path
- `Path.subpathOn_zero_one`: the full subpath [0,1] is homotopic to the original path
- Quotient-level versions of these theorems

This is split out from leanprover-community#31576 to allow independent review.

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
@github-actions
Copy link

github-actions bot commented Jan 29, 2026

PR summary 17e9ef1cfc

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.Topology.UnitInterval.ConvexSpace (new file) 1173

Declarations diff

+ coe_half
+ continuous_convexCombo
+ convexCombo
+ convexCombo_one
+ convexCombo_zero
+ convexCombo_zero_one
+ half
+ subpathOn
+ subpathOn_apply
+ subpathOn_trans_aux₁
+ subpathOn_trans_aux₂
++ convexCombo_same
++ subpathOn_self
++ subpathOn_trans
++ subpathOn_zero_one

You can run this locally as follows
## summary with just the declaration names:
./scripts/declarations_diff.sh <optional_commit>

## more verbose report:
./scripts/declarations_diff.sh long <optional_commit>

The doc-module for script/declarations_diff.sh contains some details about this script.


No changes to technical debt.

You can run this locally as

./scripts/technical-debt-metrics.sh pr_summary
  • The relative value is the weighted sum of the differences with weight given by the inverse of the current value of the statistic.
  • The absolute value is the relative value divided by the total sum of the inverses of the current values (i.e. the weighted average of the differences).

@jcommelin jcommelin added the awaiting-author A reviewer has asked the author a question or requested changes. label Jan 29, 2026
kim-em and others added 2 commits January 30, 2026 13:53
Refactors `Path.subpathOn` to use `Set.Icc.convexCombo` directly,
removing redundant inline proofs. Also adds:

- `Set.Icc.convexCombo_same`: simp lemma for `convexCombo x x t = x`
- `Set.Icc.convexCombo_zero_one`: simp lemma for endpoints
- `Set.Icc.continuous_convexCombo`: continuity with `@[fun_prop]`
- New file `Topology/UnitInterval/ConvexSpace.lean` with
  `unitInterval.convexCombo` for abstract convex spaces

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
…lemma

- Move `unitInterval.half` and `coe_half` from Path.lean to UnitInterval.lean
- Delete duplicate `continuous_convexCombo₃` (identical to `continuous_convexCombo`)

Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
@kim-em kim-em removed the awaiting-author A reviewer has asked the author a question or requested changes. label Jan 30, 2026
@jcommelin
Copy link
Member

/claude learn new skill: run lake exe mk_all after adding new files

@jcommelin jcommelin added the awaiting-author A reviewer has asked the author a question or requested changes. label Jan 30, 2026
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

awaiting-author A reviewer has asked the author a question or requested changes. t-topology Topological spaces, uniform spaces, metric spaces, filters

Projects

None yet

Development

Successfully merging this pull request may close these issues.

2 participants