Changelog

2025-01-21 14:01 6e13e010
feat: `casesm` tactic reuses hypothesis name if only one new hypothesis (#20763) …
2 files1 defs
2025-01-21 01:50 0885c937
fix: make `NNRatCast` computable for `NNReal` and `ENNReal` (#20884) …
3 files1 theorems
2025-01-21 01:50 94352f57
feat: show `IsGreatest (spectrum ℝ≥0 a) ‖a‖₊` for `IsometricContinuousFunctionalCalculus` (#20882) …
1 files14 theorems
2025-01-21 01:06 cb161584
feat: tag `csInf_insert` and `csSup_insert` `@[simp]` (#20883) …
2 files
2025-01-21 01:06 ba4ffc06
refactor(LinearAlgebra/Projection): Use IsIdempotentElem (#20665) …
4 files5 theorems
2025-01-21 01:06 0d80c6dc
chore: replace open scoped Classical with `open scoped Classical in` or `classical` (#20501) …
39 files1 theorems
2025-01-21 00:20 0371e093
feat(Logic/Basic): `HEq (cast h a) b ↔ HEq a b` (#20847) …
1 files2 theorems
2025-01-20 19:50 3c2c5041
feat(Data/Matroid/Basic): matroid congruence definitions (#20876) …
1 files3 defs
2025-01-20 18:16 ec0f40db
feat: `notation3`-defined pretty printers now make tokens that are clickable in documentation (#20861) …
2 files3 defs
2025-01-20 17:23 535a874a
feat(GroupTheory/SpecificGroups): dihedral groups are not cyclic (with one exception) (#20817)
5 files6 theorems
2025-01-20 16:38 2a250b52
fix(Linter/Style.lean): fix some outdated comments (#20879)
1 files
2025-01-20 16:38 0fecf8fc
chore(100,1000.yaml): name the authors field 'authors' (#20875) …
3 files
2025-01-20 16:38 88adf8aa
doc(Order/KrullDimension): clarify docstring of height, coheight (#20868)
1 files
2025-01-20 16:09 8f68dc48
chore: rename ENNReal lemmas to mul_{left,right}_inj for consistency (#20880)
4 files2 theorems
2025-01-20 16:09 82838c6a
feat(Data/Matroid/IndepAxioms): Another constructor for finitary matroids (#20877) …
1 files1 theorems
2025-01-20 16:09 9f8c595d
style: replace `field x y := match x, y with` with `field` (#20866) …
16 files
2025-01-20 16:09 dfa76e7f
feat(Order/Chain): adapt linear order lemmas to chains (#20757) …
1 files4 theorems
2025-01-20 16:09 4e3f39f8
feat(CategoryTheory/Localization): HasLocalization holds iff the localized category is locally small (#20670) …
2 files1 theorems
2025-01-20 16:09 80485942
feat(AlgebraicGeometry): Formally unramified morphisms (#20603)
6 files4 theorems
2025-01-20 16:09 8b8fcb5b
feat(AlgebraicGeometry): Instances regarding affine spaces (#20314)
4 files8 theorems1 defs
2025-01-20 16:09 00664149
feat(Analysis/Pow/Deriv): add some results about differentiability of cpow (#19944) …
2 files12 theorems
2025-01-20 16:09 9ebb5ca0
feat(Data/Matroid/Restrict): added a few matroid restriction lemmas (#19838) …
1 files6 theorems
2025-01-20 16:09 b823988b
feat: use to_additive for Monoid.End (#19687) …
3 files8 theorems
2025-01-20 15:19 5426682c
feat(RingTheory/Trace): the trace from a ring `R` to itself is the identity (#20865) …
1 files2 theorems
2025-01-20 15:19 fb0f8faf
chore(Algebra/CharP): `prime_ringChar` and `isPrimePow_card` (#20860) …
2 files2 theorems
2025-01-20 15:19 981f44b2
feat(RingTheory/Invariant): Galois extensions satisfy `Algebra.IsInvariant` (#20106) …
1 files1 theorems
2025-01-20 15:19 914ded28
feat: the pairs `{t, insert a t}` are pairwise disjoint (#20062) …
5 files6 theorems
2025-01-20 15:19 3f57df84
feat: Myhill–Nerode theorem (#11311) …
3 files12 theorems2 defs
2025-01-20 15:06 f033341c
feat(RingTheory): minimal primes are contained in zero divisors (#20306)
1 files3 theorems
2025-01-20 15:06 30811210
chore(Data/Matroid/Basic): a few tweaks to `Matroid.Basic` (#19836) …
3 files3 theorems
2025-01-20 13:22 3368abb8
chore(LinearAlgebra): generalize results on ranks to semirings (#20774)
11 files15 theorems1 defs
2025-01-20 13:12 b7334524
feat(CategoryTheory): localization of trifunctors (#20788) …
2 files3 theorems1 defs
2025-01-20 12:14 6313738a
feat(RingTheory/Idempotents): generalize to Semiring, add Corner and direct product decomposition (#20531) …
2 files9 theorems6 defs
2025-01-20 12:00 edaed4a2
refactor(RingTheory): split off heavy results from `Mathlib/RingTheory/Spectrum/*/Basic.lean` (#20845) …
8 files50 theorems8 defs
2025-01-20 11:48 049c0a24
feat: add lemmas for working with orders of analytic functions (#20813) …
1 files3 theorems
2025-01-20 11:48 30e9b28a
feat(RingTheory): `H¹(L)` under localization (#20591)
4 files7 theorems7 defs
2025-01-20 11:09 3bf4857a
chore(Order): split `GaloisConnection` into `Defs.lean` and `Basic.lean` (#20798) …
17 files90 theorems22 defs4 structures
2025-01-20 11:09 43e08d28
feat(BigOperators): ite_prod_one / ite_sum_zero (#20779) …
1 files2 theorems
2025-01-20 11:09 f09056ef
feat(RingTheory): prime is restriction of a prime iff it is the restriction of its extension (#20700) …
3 files4 theorems
2025-01-20 10:56 1b34e3c4
feat(RingTheory/Ideal): the height of an ideal (#20741) …
5 files19 theorems
2025-01-20 10:42 e43c7732
feat(Algebra/Category/Grp/LargeColimits): large colimits in the category of commutative additive groups (#20522) …
4 files4 theorems
2025-01-20 10:01 f68a59e8
feat: more `PGame.identical` `PGame.memₗ` `PGame.memᵣ` APIs (#5901) …
2 files25 theorems
2025-01-20 08:54 c4510a08
feat: make `Sub ℝ≥0` and `Sub ℝ≥0∞` computable (#20856) …
3 files2 defs
2025-01-20 04:58 0f52dbc8
feat: restriction of scalars for root pairings with coefficients in a field (#20384) …
5 files9 theorems1 defs
2025-01-20 04:11 510fdca8
feat(SetTheory/Order/Basic): not_lt_iff_not_le_or_ge (#19973) …
2 files1 theorems
2025-01-20 03:19 14f0a138
doc(MeasurableSpace/CountablyGenerated): fix declaration names in module doc (#20863) …
1 files
2025-01-20 01:43 f09f967a
feat: inequalities on complex exponentials (#20844) …
1 files3 theorems
2025-01-19 23:29 68ea7d25
chore(Algebra/Order/Floor): Split off `round` section (#20831) …
6 files54 theorems2 defs
2025-01-19 22:57 b13cefd9
feat: `Pi.ofNat_def` (#20857)
1 files1 theorems
2025-01-19 21:48 260650d9
feat(Order/OrderIsoNat): sequence in well-founded order is not `StrictAnti` (#20851)
1 files2 theorems