Skip to content

Commit

Permalink
bump to nightly-2023-04-07-02
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Apr 7, 2023
1 parent f6f994b commit 3f97997
Show file tree
Hide file tree
Showing 44 changed files with 519 additions and 213 deletions.
5 changes: 4 additions & 1 deletion Mathbin/Algebra/CharP/CharAndCard.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Michael Stoll
! This file was ported from Lean 3 source module algebra.char_p.char_and_card
! leanprover-community/mathlib commit 2fae5fd7f90711febdadf19c44dc60fae8834d1b
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -14,6 +14,9 @@ import Mathbin.GroupTheory.Perm.Cycle.Type
/-!
# Characteristic and cardinality
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
We prove some results relating characteristic and cardinality of finite rings
## Tags
Expand Down
1 change: 1 addition & 0 deletions Mathbin/All.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2265,6 +2265,7 @@ import Mathbin.NumberTheory.ModularForms.SlashActions
import Mathbin.NumberTheory.ModularForms.SlashInvariantForms
import Mathbin.NumberTheory.Multiplicity
import Mathbin.NumberTheory.NumberField.Basic
import Mathbin.NumberTheory.NumberField.CanonicalEmbedding
import Mathbin.NumberTheory.NumberField.ClassNumber
import Mathbin.NumberTheory.NumberField.Embeddings
import Mathbin.NumberTheory.NumberField.Norm
Expand Down
4 changes: 2 additions & 2 deletions Mathbin/Analysis/InnerProductSpace/Projection.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Zhouhang Zhou, Frédéric Dupuis, Heather Macbeth
! This file was ported from Lean 3 source module analysis.inner_product_space.projection
! leanprover-community/mathlib commit 039a089d2a4b93c761b234f3e5f5aeb752bac60f
! leanprover-community/mathlib commit 67e606eaea14c7854bdc556bd53d98aefdf76ec0
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down Expand Up @@ -1171,7 +1171,7 @@ theorem Submodule.finrank_add_inf_finrank_orthogonal {K₁ K₂ : Submodule 𝕜
by
haveI := Submodule.finiteDimensional_of_le h
haveI := proper_is_R_or_C 𝕜 K₁
have hd := Submodule.rank_sup_add_rank_inf_eq K₁ (K₁ᗮ ⊓ K₂)
have hd := Submodule.finrank_sup_add_finrank_inf_eq K₁ (K₁ᗮ ⊓ K₂)
rw [← inf_assoc, (Submodule.orthogonal_disjoint K₁).eq_bot, bot_inf_eq, finrank_bot,
Submodule.sup_orthogonal_inf_of_completeSpace h] at hd
rw [add_zero] at hd
Expand Down
6 changes: 3 additions & 3 deletions Mathbin/Analysis/NormedSpace/FiniteDimension.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sébastien Gouëzel
! This file was ported from Lean 3 source module analysis.normed_space.finite_dimension
! leanprover-community/mathlib commit be2ac64be57e8319fcd5c5547f3a8d9412daf5ec
! leanprover-community/mathlib commit 5ec62c8106221a3f9160e4e4fcc3eed79fe213e9
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down Expand Up @@ -440,7 +440,7 @@ variable (𝕜 E)

theorem FiniteDimensional.complete [FiniteDimensional 𝕜 E] : CompleteSpace E :=
by
set e := ContinuousLinearEquiv.ofFinrankEq (@finrank_fin_fun 𝕜 _ (finrank 𝕜 E)).symm
set e := ContinuousLinearEquiv.ofFinrankEq (@finrank_fin_fun 𝕜 _ _ (finrank 𝕜 E)).symm
have : UniformEmbedding e.to_linear_equiv.to_equiv.symm := e.symm.uniform_embedding
exact (completeSpace_congr this).1 (by infer_instance)
#align finite_dimensional.complete FiniteDimensional.complete
Expand Down Expand Up @@ -692,7 +692,7 @@ properness of `𝕜`, and the search for `𝕜` as an unknown metavariable. Decl
explicitly when needed. -/
theorem FiniteDimensional.proper [FiniteDimensional 𝕜 E] : ProperSpace E :=
by
set e := ContinuousLinearEquiv.ofFinrankEq (@finrank_fin_fun 𝕜 _ (finrank 𝕜 E)).symm
set e := ContinuousLinearEquiv.ofFinrankEq (@finrank_fin_fun 𝕜 _ _ (finrank 𝕜 E)).symm
exact e.symm.antilipschitz.proper_space e.symm.continuous e.symm.surjective
#align finite_dimensional.proper FiniteDimensional.proper

Expand Down
5 changes: 4 additions & 1 deletion Mathbin/CategoryTheory/Abelian/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Markus Himmel, Johan Commelin, Scott Morrison
! This file was ported from Lean 3 source module category_theory.abelian.basic
! leanprover-community/mathlib commit 8c75ef3517d4106e89fe524e6281d0b0545f47fc
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -17,6 +17,9 @@ import Mathbin.CategoryTheory.Abelian.NonPreadditive
/-!
# Abelian categories
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file contains the definition and basic properties of abelian categories.
There are many definitions of abelian category. Our definition is as follows:
Expand Down
5 changes: 4 additions & 1 deletion Mathbin/CategoryTheory/Grothendieck.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison

! This file was ported from Lean 3 source module category_theory.grothendieck
! leanprover-community/mathlib commit 14b69e9f3c16630440a2cbd46f1ddad0d561dee7
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -14,6 +14,9 @@ import Mathbin.CategoryTheory.Elements
/-!
# The Grothendieck construction

> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.

Given a functor `F : C ⥤ Cat`, the objects of `grothendieck F`
consist of dependent pairs `(b, f)`, where `b : C` and `f : F.obj c`,
and a morphism `(b, f) ⟶ (b', f')` is a pair `β : b ⟶ b'` in `C`, and
Expand Down
7 changes: 3 additions & 4 deletions Mathbin/CategoryTheory/Preadditive/Schur.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Markus Himmel, Scott Morrison
! This file was ported from Lean 3 source module category_theory.preadditive.schur
! leanprover-community/mathlib commit 829895f162a1f29d0133f4b3538f4cd1fb5bffd3
! leanprover-community/mathlib commit 5ec62c8106221a3f9160e4e4fcc3eed79fe213e9
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down Expand Up @@ -126,8 +126,7 @@ theorem finrank_endomorphism_eq_one {X : C} (is_iso_iff_nonzero : ∀ f : X ⟶
[I : FiniteDimensional 𝕜 (X ⟶ X)] : finrank 𝕜 (X ⟶ X) = 1 :=
by
have id_nonzero := (is_iso_iff_nonzero (𝟙 X)).mp (by infer_instance)
apply finrank_eq_one (𝟙 X)
· exact id_nonzero
refine' finrank_eq_one (𝟙 X) id_nonzero _
· intro f
haveI : Nontrivial (End X) := nontrivial_of_ne _ _ id_nonzero
obtain ⟨c, nu⟩ :=
Expand Down Expand Up @@ -191,7 +190,7 @@ theorem finrank_hom_simple_simple_le_one (X Y : C) [FiniteDimensional 𝕜 (X
exact zero_le_one
· obtain ⟨f, nz⟩ := (nontrivial_iff_exists_ne 0).mp h
haveI fi := (is_iso_iff_nonzero f).mpr nz
apply finrank_le_one f
refine' finrank_le_one f _
intro g
obtain ⟨c, w⟩ := endomorphism_simple_eq_smul_id 𝕜 (g ≫ inv f)
exact ⟨c, by simpa using w =≫ f⟩
Expand Down
5 changes: 4 additions & 1 deletion Mathbin/CategoryTheory/Sites/Sheaf.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard, Bhavik Mehta

! This file was ported from Lean 3 source module category_theory.sites.sheaf
! leanprover-community/mathlib commit a67ec23dd8dc08195d77b6df2cd21f9c64989131
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -17,6 +17,9 @@ import Mathbin.CategoryTheory.Sites.SheafOfTypes
/-!
# Sheaves taking values in a category

> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.

If C is a category with a Grothendieck topology, we define the notion of a sheaf taking values in
an arbitrary category `A`. We follow the definition in https://stacks.math.columbia.edu/tag/00VR,
noting that the presheaf of sets "defined above" can be seen in the comments between tags 00VQ and
Expand Down
5 changes: 4 additions & 1 deletion Mathbin/Combinatorics/SimpleGraph/AdjMatrix.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Aaron Anderson, Jalex Stark, Kyle Miller, Lu-Ming Zhang
! This file was ported from Lean 3 source module combinatorics.simple_graph.adj_matrix
! leanprover-community/mathlib commit 3e068ece210655b7b9a9477c3aff38a492400aa1
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -16,6 +16,9 @@ import Mathbin.LinearAlgebra.Matrix.Symmetric
/-!
# Adjacency Matrices
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This module defines the adjacency matrix of a graph, and provides theorems connecting graph
properties to computational properties of the matrix.
Expand Down
5 changes: 4 additions & 1 deletion Mathbin/Combinatorics/SimpleGraph/IncMatrix.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Moise, Yaël Dillies, Kyle Miller
! This file was ported from Lean 3 source module combinatorics.simple_graph.inc_matrix
! leanprover-community/mathlib commit bb168510ef455e9280a152e7f31673cabd3d7496
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -14,6 +14,9 @@ import Mathbin.Data.Matrix.Basic
/-!
# Incidence matrix of a simple graph
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines the unoriented incidence matrix of a simple graph.
## Main definitions
Expand Down
5 changes: 4 additions & 1 deletion Mathbin/Computability/Ackermann.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Violeta Hernández Palacios
! This file was ported from Lean 3 source module computability.ackermann
! leanprover-community/mathlib commit 9b2660e1b25419042c8da10bf411aa3c67f14383
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -14,6 +14,9 @@ import Mathbin.Tactic.Linarith.Default
/-!
# Ackermann function
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file, we define the two-argument Ackermann function `ack`. Despite having a recursive
definition, we show that this isn't a primitive recursive function.
Expand Down
4 changes: 2 additions & 2 deletions Mathbin/Data/Finset/Basic.lean

Large diffs are not rendered by default.

4 changes: 2 additions & 2 deletions Mathbin/Data/Finset/Image.lean

Large diffs are not rendered by default.

5 changes: 4 additions & 1 deletion Mathbin/Data/String/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
! This file was ported from Lean 3 source module data.string.basic
! leanprover-community/mathlib commit d13b3a4a392ea7273dfa4727dbd1892e26cfd518
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -14,6 +14,9 @@ import Mathbin.Data.Char
/-!
# Strings
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Supplementary theorems about the `string` type.
-/

Expand Down
5 changes: 2 additions & 3 deletions Mathbin/FieldTheory/Finite/Polynomial.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johan Commelin
! This file was ported from Lean 3 source module field_theory.finite.polynomial
! leanprover-community/mathlib commit 039a089d2a4b93c761b234f3e5f5aeb752bac60f
! leanprover-community/mathlib commit 5aa3c1de9f3c642eac76e11071c852766f220fd0
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down Expand Up @@ -217,8 +217,7 @@ theorem rank_r [Fintype σ] : Module.rank K (R σ K) = Fintype.card (σ → K) :
Module.rank K (↥{ s : σ →₀ ℕ | ∀ n : σ, s n ≤ Fintype.card K - 1 } →₀ K) :=
LinearEquiv.rank_eq
(Finsupp.supportedEquivFinsupp { s : σ →₀ ℕ | ∀ n : σ, s n ≤ Fintype.card K - 1 })
_ = (#{ s : σ →₀ ℕ | ∀ n : σ, s n ≤ Fintype.card K - 1 }) := by
rw [Finsupp.rank_eq, rank_self, mul_one]
_ = (#{ s : σ →₀ ℕ | ∀ n : σ, s n ≤ Fintype.card K - 1 }) := by rw [rank_finsupp_self']
_ = (#{ s : σ → ℕ | ∀ n : σ, s n < Fintype.card K }) :=
by
refine' Quotient.sound ⟨Equiv.subtypeEquiv Finsupp.equivFunOnFinite fun f => _⟩
Expand Down
5 changes: 4 additions & 1 deletion Mathbin/GroupTheory/Perm/Cycle/Type.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Thomas Browning
! This file was ported from Lean 3 source module group_theory.perm.cycle.type
! leanprover-community/mathlib commit 47adfab39a11a072db552f47594bf8ed2cf8a722
! leanprover-community/mathlib commit 75be6b616681ab6ca66d798ead117e75cd64f125
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -18,6 +18,9 @@ import Mathbin.Tactic.Linarith.Default
/-!
# Cycle Types
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file we define the cycle type of a permutation.
## Main definitions
Expand Down
4 changes: 2 additions & 2 deletions Mathbin/LinearAlgebra/AffineSpace/FiniteDimensional.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Myers
! This file was ported from Lean 3 source module linear_algebra.affine_space.finite_dimensional
! leanprover-community/mathlib commit 039a089d2a4b93c761b234f3e5f5aeb752bac60f
! leanprover-community/mathlib commit 67e606eaea14c7854bdc556bd53d98aefdf76ec0
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down Expand Up @@ -735,7 +735,7 @@ theorem finrank_vectorSpan_insert_le (s : AffineSubspace k P) (p : P) :
rw [← finrank_bot k V]
convert rfl <;> simp
· rw [affine_span_coe, direction_affine_span_insert hp₀, add_comm]
refine' (Submodule.rank_add_le_rank_add_rank _ _).trans (add_le_add_right _ _)
refine' (Submodule.finrank_add_le_finrank_add_finrank _ _).trans (add_le_add_right _ _)
refine' finrank_le_one ⟨p -ᵥ p₀, Submodule.mem_span_singleton_self _⟩ fun v => _
have h := v.property
rw [Submodule.mem_span_singleton] at h
Expand Down
4 changes: 2 additions & 2 deletions Mathbin/LinearAlgebra/BilinearForm.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Andreas Swerdlow, Kexing Ying
! This file was ported from Lean 3 source module linear_algebra.bilinear_form
! leanprover-community/mathlib commit 039a089d2a4b93c761b234f3e5f5aeb752bac60f
! leanprover-community/mathlib commit 67e606eaea14c7854bdc556bd53d98aefdf76ec0
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down Expand Up @@ -1479,7 +1479,7 @@ theorem restrict_nondegenerate_of_isCompl_orthogonal {B : BilinForm K V} {W : Su
exact hx₂ n hn
refine' IsCompl.of_eq this (eq_top_of_finrank_eq <| (Submodule.finrank_le _).antisymm _)
conv_rhs => rw [← add_zero (finrank K _)]
rw [← finrank_bot K V, ← this, Submodule.rank_sup_add_rank_inf_eq,
rw [← finrank_bot K V, ← this, Submodule.finrank_sup_add_finrank_inf_eq,
finrank_add_finrank_orthogonal b₁]
exact le_self_add
#align bilin_form.restrict_nondegenerate_of_is_compl_orthogonal BilinForm.restrict_nondegenerate_of_isCompl_orthogonal
Expand Down
Loading

0 comments on commit 3f97997

Please sign in to comment.