mathlib icon indicating copy to clipboard operation
mathlib copied to clipboard

Lean 3's obsolete mathematical components library: please use mathlib4

Results 381 mathlib issues
Sort by recently updated
recently updated
newest added

Informally, this is the "minimum distance", though "minimum" makes sense mainly only in the finite context. This is analogous to diam in some sense. We provide finset and set versions...

awaiting-review
t-topology

* The new `cont_diff_within_at_succ_iff_has_fderiv_within_at'` generalizes `cont_diff_within_at.has_fderiv_within_at_nhds` and `cont_diff_within_at_succ_iff_has_fderiv_within_at_of_mem` * Prove that `has_fderiv_within_at` and `cont_diff_within_at` are not dependent on adding a single point to the set * Add some more lemmas...

awaiting-review
t-analysis

This splits `data.set.pointwise` and `data.finset.pointwise` each into several smaller files. This allows us to remove or defer some imports, e.g. of `order.well_founded_set` and of `algebra.big_operators.basic`. No changes to statements of...

awaiting-review
awaiting-CI

Proof by induction on the number of summands. finset.sym is used to sum over. It means we have access to the finset tooling to rewrite it, and it's one of...

awaiting-review
blocked-by-other-PR
t-algebra
t-combinatorics

Add lemmas that, in a real normed space, the sets of points on the same side of an affine subspace as a given point, or on the opposite side from...

awaiting-author

This PR defines triangular matrices based on block-triangular matrices. --- - [x] depends on: #14035 - [x] depends on: #16150 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

Add a definition of (bundled) subgroupoid and prove some of their basic properties. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
t-algebra

--- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
t-order

In this PR we define the conductor ideal and prove some basic results about it. In a later PR (#16870), these will be used to prove the Dedekind-Kummer theorem in...

awaiting-review

--- See also comments [on Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/ideals.20in.20non-comm.20rings/near/284039475) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

please-adopt
too-late