Skip to content

Commit

Permalink
bump
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Apr 22, 2024
1 parent fc9d94c commit f939c87
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion FltRegular/FltThree/Spts.lean
Original file line number Diff line number Diff line change
Expand Up @@ -396,7 +396,7 @@ theorem Spts.four {p : ℤ√(-3)} (hfour : p.norm = 4) (hq : p.im ≠ 0) : abs
ring

· rw [← Int.sub_one_lt_iff, sub_self]
exact sq_pos_of_ne_zero _ hq
exact sq_pos_of_ne_zero hq
refine' ⟨_, hq⟩
calc
p.re ^ 2 = p.re ^ 2 + 3 * p.im ^ 2 - 3 := by simp [hq]
Expand Down
4 changes: 2 additions & 2 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": "32983874c1b897d78f20d620fe92fc8fd3f06c3a",
"rev": "e840c18f7334c751efbd4cfe531476e10c943cdb",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand Down Expand Up @@ -58,7 +58,7 @@
{"url": "https://github.com/leanprover-community/mathlib4.git",
"type": "git",
"subDir": null,
"rev": "145460b9327f120bf7013552bb8e8185bd226dea",
"rev": "cc96d0afe2eefff4ef1ca9e065eed50c34d775c8",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
Expand Down

0 comments on commit f939c87

Please sign in to comment.