Skip to content

Commit

Permalink
bump
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Mar 17, 2024
1 parent cafcac5 commit 3ee4681
Show file tree
Hide file tree
Showing 2 changed files with 9 additions and 9 deletions.
8 changes: 4 additions & 4 deletions FltRegular/FltThree/OddPrimeOrFour.lean
Original file line number Diff line number Diff line change
Expand Up @@ -117,8 +117,8 @@ theorem factors_unique_prod' :
noncomputable def oddFactors (x : ℕ) :=
Multiset.filter Odd (UniqueFactorizationMonoid.normalizedFactors x)

theorem oddFactors.zero : oddFactors 0 = 0 :=
rfl
theorem oddFactors.zero : oddFactors 0 = 0 := by
simp [oddFactors]

theorem oddFactors.not_two_mem (x : ℕ) : 2 ∉ oddFactors x := by
simp [oddFactors]
Expand All @@ -136,8 +136,8 @@ theorem evenFactorExp.def (x : ℕ) :
evenFactorExp x = Multiset.count 2 (UniqueFactorizationMonoid.normalizedFactors x) :=
rfl

theorem evenFactorExp.zero : evenFactorExp 0 = 0 :=
rfl
theorem evenFactorExp.zero : evenFactorExp 0 = 0 := by
simp [evenFactorExp]

theorem evenFactorExp.pow (z : ℕ) (n : ℕ) : evenFactorExp (z ^ n) = n * evenFactorExp z :=
by
Expand Down
10 changes: 5 additions & 5 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "ff9850c4726f6b9fb8d8e96980c3fcb2900be8bd",
"rev": "f3447c3732c9d6e8df3bdad78e5ecf7e8b353bbc",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -22,7 +22,7 @@
{"url": "https://github.com/leanprover-community/aesop",
"type": "git",
"subDir": null,
"rev": "056ca0fa8f5585539d0b940f532d9750c3a2270f",
"rev": "8be30c25e3caa06937feeb62f7ca898370f80ee9",
"name": "aesop",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
Expand All @@ -40,7 +40,7 @@
{"url": "https://github.com/leanprover/lean4-cli",
"type": "git",
"subDir": null,
"rev": "a751d21d4b68c999accb6fc5d960538af26ad5ec",
"rev": "be8fa79a28b8b6897dce0713ef50e89c4a0f6ef5",
"name": "Cli",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -49,7 +49,7 @@
{"url": "https://github.com/leanprover-community/import-graph.git",
"type": "git",
"subDir": null,
"rev": "64d082eeaad1a8e6bbb7c23b7a16b85a1715a02f",
"rev": "bbcffbcc19d69e13d5eea716283c76169db524ba",
"name": "importGraph",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -58,7 +58,7 @@
{"url": "https://github.com/leanprover-community/mathlib4.git",
"type": "git",
"subDir": null,
"rev": "f884087a041da7998696e87352f6f06e2e5f5713",
"rev": "6d1dffa1281a6e231f594e4c49ec01bc3ad9974e",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
Expand Down

0 comments on commit 3ee4681

Please sign in to comment.