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

This PR defines 1. the `sup_degree` of an `add_monoid_algebra`, graded by a `semilattice_sup`; 1. the `inf_degree` of an `add_monoid_algebra`, graded by a `semilattice_inf`; 1. the `max_degree` of an `add_monoid_algebra`, graded...

awaiting-review

* Remove the `t2_space` assumption from `exists_compact_between` by generalizing the proof of `exists_compact_superset`, and move it from `topology/separation` to `topology/subset_properties`. * Use it to prove `continuous_map.continuous_prod` in `topology/continuous_map` stating that...

awaiting-review
t-topology

Define `real.angle.to_real`, converting a `real.angle` to a real in the interval `Ioc (-π) π` (the same interval used by `complex.arg`), and prove some associated lemmas. This is the inverse operation...

awaiting-review
t-analysis

This contains the definition of a congruence subgroup of `SL(2,Z)` and defines Gamma1, Gamma0 and full level subgroups. It also contains some basic results about them. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review

The defines the notion of functions on the upper half plane being bounded at infinity and zero at infinity. This is required for #13250. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review

Define the property of being triangle-free far. This comes up in the triangle counting and triangle removal lemmas. Co-authored-by: Bhavik Mehta --- - [x] depends on: #12982 - [x] depends...

awaiting-review

Lean is unable to automatically infer `ordered_smul` instance for `fin n → ℝ` from [docs#ordered_smul'](https://leanprover-community.github.io/mathlib_docs/algebra/order/module.html#pi.ordered_smul'). This in turns leads to issues with defining the [docs#convex_cone.positive](https://leanprover-community.github.io/mathlib_docs/find/convex_cone.positive) in these vector spaces. [Zulip...

bug
WIP

Proof that the dual of dual of a closed convex cone is itself. I'll break this result into smaller PRs. This result is fundamental to formalising linear (or rather conic)...

awaiting-review
t-analysis

The six lemmas in this PR show that * `finset.max` and `finset.max'` coincide (when and how they can); * the `finset.max'` of `s.erase x` is not `x`; * the `finset.max`...

awaiting-review

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

awaiting-review