Skip to content

Commit f939c87

Browse files
bump
1 parent fc9d94c commit f939c87

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

FltRegular/FltThree/Spts.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -396,7 +396,7 @@ theorem Spts.four {p : ℤ√(-3)} (hfour : p.norm = 4) (hq : p.im ≠ 0) : abs
396396
ring
397397

398398
· rw [← Int.sub_one_lt_iff, sub_self]
399-
exact sq_pos_of_ne_zero _ hq
399+
exact sq_pos_of_ne_zero hq
400400
refine' ⟨_, hq⟩
401401
calc
402402
p.re ^ 2 = p.re ^ 2 + 3 * p.im ^ 2 - 3 := by simp [hq]

lake-manifest.json

+2-2
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@
44
[{"url": "https://github.com/leanprover/std4",
55
"type": "git",
66
"subDir": null,
7-
"rev": "32983874c1b897d78f20d620fe92fc8fd3f06c3a",
7+
"rev": "e840c18f7334c751efbd4cfe531476e10c943cdb",
88
"name": "std",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",
@@ -58,7 +58,7 @@
5858
{"url": "https://github.com/leanprover-community/mathlib4.git",
5959
"type": "git",
6060
"subDir": null,
61-
"rev": "145460b9327f120bf7013552bb8e8185bd226dea",
61+
"rev": "cc96d0afe2eefff4ef1ca9e065eed50c34d775c8",
6262
"name": "mathlib",
6363
"manifestFile": "lake-manifest.json",
6464
"inputRev": null,

0 commit comments

Comments
 (0)