-
Notifications
You must be signed in to change notification settings - Fork 356
Commit
This commit does not belong to any branch on this repository, and may belong to a fork outside of the repository.
chore: bump Std, changes for leanprover-community/batteries#366
revert . fix a bit blech one more comment out broken and unused results chore: bump Std remove redundant simp lemmas cleanup fix: make `Nat.testBit_bitwise` a simp-lemma again. This fixes the Int.testbit_bitwise proofs fix `castNum_testBit` fix `testBit_eq_inth` fixes golf golf Apply suggestions from code review Co-authored-by: Eric Wieser <[email protected]> fix whitespace fix name conflict more efficient restore lemma feat: Mapping extreme points under continuous maps (#8574) Prove that extreme points are preserved under affine equivalences, and the less trivial statement that a continuous affine map sends extreme points of a compact set to a superset of the extreme points of the image of that set. Also fix a few name and tweak the API a bit. Co-authored-by: Yury G. Kudryashov <[email protected]> chore(Profinite): allow more universe flexibility in Profinite/CofilteredLimit (#8613) We allow the indexing category for the cofiltered limit in the result `Profinite.exists_locallyConstant` to live in a smaller universe than our profinite sets. feat(CategoryTheory): `Preregular` and `FinitaryPreExtensive` implies `Precoherent` (#8643) We prove some results about effective epimorphisms which allow us to deduce that a category which is `FinitaryPreExtensive` and `Preregular`Β is also `Precoherent`. feat(Analysis/Seminorm): add more `*ball_smul_*ball` (#8724) We had `ball_smul_ball` and `closedBall_smul_closedBall`. Add versions with mixed `ball` and `closedBall`. Also move this lemmas below and golf the proofs. feat: the annihilator of the kernel of the trace form of a Lie module is contained in the span of its weights (#8739) fix breakage in BitVec lemmas
- Loading branch information
1 parent
6f22008
commit 7cd93d7
Showing
26 changed files
with
437 additions
and
286 deletions.
There are no files selected for viewing
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Oops, something went wrong.