Skip to content

Commit

Permalink
bump to nightly-2023-03-01-00
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Mar 1, 2023
1 parent 1fb1623 commit bccc50c
Show file tree
Hide file tree
Showing 10 changed files with 161 additions and 163 deletions.
4 changes: 2 additions & 2 deletions Mathbin/Algebra/Group/Units.lean
Original file line number Diff line number Diff line change
Expand Up @@ -125,9 +125,9 @@ def [anonymous] (u : αˣ) : α :=
↑u⁻¹
#align units.simps.coe_inv [anonymous]
initialize_simps_projections Units (val → coe as_prefix, inv → coe_inv as_prefix)
initialize_simps_projections Units (val → coe, as_prefix coe, inv → coe_inv, as_prefix coe_inv)
initialize_simps_projections AddUnits (val → coe as_prefix, neg → coe_neg as_prefix)
initialize_simps_projections AddUnits (val → coe, as_prefix coe, neg → coe_neg, as_prefix coe_neg)
/- warning: units.coe_mk -> Units.val_mk is a dubious translation:
lean 3 declaration is
Expand Down
2 changes: 1 addition & 1 deletion Mathbin/Algebra/Module/Equiv.lean

Large diffs are not rendered by default.

2 changes: 1 addition & 1 deletion Mathbin/LinearAlgebra/AffineSpace/AffineEquiv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -214,7 +214,7 @@ def Simps.symmApply (e : P₁ ≃ᵃ[k] P₂) : P₂ → P₁ :=
#align affine_equiv.simps.symm_apply AffineEquiv.Simps.symmApply

initialize_simps_projections AffineEquiv (to_equiv_to_fun → apply, to_equiv_inv_fun → symm_apply,
linear → linear as_prefix, -toEquiv)
linear → linear, as_prefix linear, -toEquiv)

protected theorem bijective (e : P₁ ≃ᵃ[k] P₂) : Bijective e :=
e.toEquiv.Bijective
Expand Down
6 changes: 3 additions & 3 deletions Mathbin/LinearAlgebra/Pi.lean

Large diffs are not rendered by default.

72 changes: 36 additions & 36 deletions Mathbin/Order/Heyting/Hom.lean

Large diffs are not rendered by default.

192 changes: 96 additions & 96 deletions Mathbin/Order/Hom/Lattice.lean

Large diffs are not rendered by default.

32 changes: 16 additions & 16 deletions Mathbin/Order/Ideal.lean

Large diffs are not rendered by default.

2 changes: 0 additions & 2 deletions Mathbin/Tactic/Simps.lean
Original file line number Diff line number Diff line change
Expand Up @@ -116,13 +116,11 @@ unsafe instance : has_to_format parsed_projection_data :=

end

#print ProjectionRule /-
/-- The type of rules that specify how metadata for projections in changes.
See `initialize_simps_projection`. -/
abbrev ProjectionRule :=
Sum (Name × Name) Name × Bool
#align projection_rule ProjectionRule
-/

/-- The `@[_simps_str]` attribute specifies the preferred projections of the given structure,
used by the `@[simps]` attribute.
Expand Down
8 changes: 4 additions & 4 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,15 +4,15 @@
[{"git":
{"url": "https://github.com/leanprover-community/lean3port.git",
"subDir?": null,
"rev": "232aaddfaaa7d23f96af916f60d521e4405b67dd",
"rev": "339fa1901df2c7f00338edf9590d8dff4f5a2974",
"name": "lean3port",
"inputRev?": "232aaddfaaa7d23f96af916f60d521e4405b67dd"}},
"inputRev?": "339fa1901df2c7f00338edf9590d8dff4f5a2974"}},
{"git":
{"url": "https://github.com/leanprover-community/mathlib4.git",
"subDir?": null,
"rev": "7b5ca5d34639cc7c0cbf129b4dedefb79fb84ec8",
"rev": "b21620a738bdb033f8e5b97ca769d89ae650bfbc",
"name": "mathlib",
"inputRev?": "7b5ca5d34639cc7c0cbf129b4dedefb79fb84ec8"}},
"inputRev?": "b21620a738bdb033f8e5b97ca769d89ae650bfbc"}},
{"git":
{"url": "https://github.com/gebner/quote4",
"subDir?": null,
Expand Down
4 changes: 2 additions & 2 deletions lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ open Lake DSL System
-- Usually the `tag` will be of the form `nightly-2021-11-22`.
-- If you would like to use an artifact from a PR build,
-- it will be of the form `pr-branchname-sha`.
def tag : String := "nightly-2023-02-28-22"
def tag : String := "nightly-2023-03-01-00"
def releaseRepo : String := "leanprover-community/mathport"
def oleanTarName : String := "mathlib3-binport.tar.gz"

Expand Down Expand Up @@ -38,7 +38,7 @@ target fetchOleans (_pkg : Package) : Unit := do
untarReleaseArtifact releaseRepo tag oleanTarName libDir
return .nil

require lean3port from git "https://github.com/leanprover-community/lean3port.git"@"232aaddfaaa7d23f96af916f60d521e4405b67dd"
require lean3port from git "https://github.com/leanprover-community/lean3port.git"@"339fa1901df2c7f00338edf9590d8dff4f5a2974"

@[default_target]
lean_lib Mathbin where
Expand Down

0 comments on commit bccc50c

Please sign in to comment.