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

Reported by @RemyDegenne on [Zulip](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/expand_exists.20questions): > I am testing the new `expand_exists` attribute, which looks like a very useful tool, and I have two remarks/questions: > - The names given...

t-meta

We have the definition of locally convex spaces and the characterization of locally convex spaces via seminorms. We have all the ingredients to prove the very useful lemma: Let X...

feature-request
good-first-project

- [x] finite - [x] finitely generated (done for submodules, we might want a wrapper to make life easier when working with a full module) (#4634) - [ ] finitely...

feature-request

We are missing instances `add_submonoid_class S M → has_coe S (add_submonoid M)` (probably `has_coe_t` now that I think of it), so we can just use `coe` [here](https://github.com/leanprover-community/mathlib/pull/14583#discussion_r907373588_). Similar coercions should...

Example ```lean import tactic.apply import data.set.basic example {α : Type*} (a b : set α) : a ⊆ b := by refl' -- closes the goal -- by apply' set.subset.refl...

bug
t-meta

In the following example, `nth_rewrite` incorrectly instantiates the universe metavariable of `h` with `0`, but still rewrites with the hypothesis. Note that `rw` does this correctly. ```lean def foo (h...

bug
t-meta

PR #11246 defines `real.logb`: the logarithm base `b`. Many lemmas about this are provided in `analysis/special_functions/logb.lean`, roughly analogous to the lemmas for the natural logarithm in `analysis/special_functions/log.lean`. But lemmas about...

feature-request
good-first-project

I don't know anything about the implementation of `norm_num`, but in my ideal world, these lemmas would entirely be handled by `norm_num`. _Originally posted by @Smaug123 in https://github.com/leanprover-community/mathlib/issues/8002#issuecomment-1158021087_ There are...

feature-request

[The long line](https://en.wikipedia.org/wiki/Long_line_(topology)) is often used as a counterexample in topology. It can be defined as `lex ℝ (Ico (0 : ℝ) 1)` which is already equipped with its order...

good-first-project

Although `fintype` and `decidable` are (sub)singletons, since different instances are not definitionally equal, it's useful to have instance arguments that are seemingly redundant. For example: ```lean lemma to_finset_inter {α :...