Skip to content

Commit 8a32b04

Browse files
committed
bump to v4.20.1
1 parent 63b51e8 commit 8a32b04

File tree

12 files changed

+30
-30
lines changed

12 files changed

+30
-30
lines changed

FormalConjectures/ErdosProblems/304.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -44,7 +44,7 @@ lemma unitFractionExpressible_of_zero {a b : ℕ} (h : a = 0 ∨ b = 0) :
4444
rintro _ s rfl hs h
4545
rw [eq_comm, Finset.sum_eq_zero_iff_of_nonneg (fun i hi ↦ by positivity)] at h
4646
simp only [inv_eq_zero, Nat.cast_eq_zero] at h
47-
rw [Finset.card_eq_zero, Finset.eq_empty_iff_forall_not_mem]
47+
rw [Finset.card_eq_zero, Finset.eq_empty_iff_forall_notMem]
4848
intro i hi
4949
linarith [h i hi, hs i hi]
5050

@@ -121,7 +121,7 @@ lemma dvd_of_smallestCollection_eq_one {a b : ℕ}
121121
lemma smallestCollection_two_fifteen : smallestCollection 2 15 = 2 := by
122122
have h : 2 ∈ unitFractionExpressible 2 15 := by
123123
use {10, 30}
124-
norm_num [Finset.card_insert_of_not_mem, Finset.card_singleton]
124+
norm_num [Finset.card_insert_of_notMem, Finset.card_singleton]
125125
have : smallestCollection 2 152 := Nat.sInf_le h
126126
have : 0 < smallestCollection 2 15 := smallestCollection_pos (by simp) (by simp) ⟨_, h⟩
127127
have : smallestCollection 2 151 := by

FormalConjectures/ForMathlib/Combinatorics/AP/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -67,7 +67,7 @@ theorem Set.isAPOfLengthWith_pair {α : Type*} [DecidableEq α] [AddCommGroup α
6767
{a b : α} (hab : a ≠ b) :
6868
Set.IsAPOfLengthWith {a, b} 2 a (b - a) := by
6969
simp [IsAPOfLengthWith]
70-
rw [Finset.card_insert_of_not_mem (by simpa only [Finset.mem_singleton])]
70+
rw [Finset.card_insert_of_notMem (by simpa only [Finset.mem_singleton])]
7171
simp
7272
refine Set.ext fun x => ⟨fun h ↦ ?_, fun ⟨n, ⟨_, _⟩⟩ ↦ by interval_cases n <;> simp_all⟩
7373
cases h with

FormalConjectures/ForMathlib/Test/Computability/TuringMachine.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -45,7 +45,7 @@ match l with
4545
instance : alwaysHaltingMachine.IsHalting where
4646
halts := by
4747
simp_rw (config := { singlePass := true })
48-
[BusyBeaver.eval, Turing.eval, Part.map_Dom, step, alwaysHaltingMachine, Option.map_none',
48+
[BusyBeaver.eval, Turing.eval, Part.map_Dom, step, alwaysHaltingMachine, Option.map_none,
4949
Part.dom_iff_mem, PFun.mem_fix_iff, Part.mem_some_iff]
5050
use default
5151
aesop

FormalConjectures/Paper/Kurepa.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -89,7 +89,7 @@ theorem kurepa_conjecture.variant.gcd (n : ℕ) : 2 < n → (n !).gcd (! n) = 2
8989
theorem kurepa_conjecture.gcd_reduction : (∀ n, 2 < n → (!n : ℕ) % n ≠ 0)
9090
↔ (∀ n, 2 < n → (n)!.gcd (!n) = 2) := by
9191
refine ⟨fun h n hn ↦ match n with | S + 1 => gcd_eq_iff.2 ?_,
92-
fun h n hn _ ↦ n.not_dvd_of_pos_of_lt (by omega) hn <| h n hn ▸ n.dvd_gcd
92+
fun h n hn _ ↦ Nat.not_dvd_of_pos_of_lt (by omega) hn <| h n hn ▸ n.dvd_gcd
9393
(n.dvd_factorial hn.pos le_rfl) (dvd_of_mod_eq_zero ‹_›)⟩
9494
refine ⟨Nat.factorial_dvd_factorial hn.le, ?_, fun c hc h_dvd ↦ ?_⟩
9595
· match S with

FormalConjectures/Wikipedia/Conway99Graph.lean

Lines changed: 6 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -25,7 +25,12 @@ import FormalConjectures.Util.ProblemImports
2525
Conway's 99-graph problem
2626
-/
2727
--TODO(firsching): Consider using SimpleGraph.IsSRGWith to formulate the conjecture.
28+
29+
open SimpleGraph
30+
2831
variable {V : Type} {G : SimpleGraph V}
32+
33+
2934
@[category undergraduate, AMS 5]
3035
lemma completeGraphIsClique (s : Finset V) : (⊤ : SimpleGraph V).IsClique s :=
3136
Pairwise.set_pairwise (fun _ _ a ↦ a) _
@@ -104,7 +109,7 @@ example : NonEdgesAreDiagonals Conway9 := by
104109
have ⟨x1, x2⟩ := x
105110
have ⟨y1, y2⟩ := y
106111
simp only [Conway9, SimpleGraph.completeGraph_eq_top,
107-
SimpleGraph.boxProd_adj, SimpleGraph.top_adj, SimpleGraph.boxProd_neighborFinset]
112+
SimpleGraph.boxProd_adj, SimpleGraph.top_adj, SimpleGraph.neighborFinset_boxProd]
108113
fin_cases x1 <;> fin_cases x2 <;> fin_cases y1 <;> fin_cases y2 <;> decide
109114

110115
@[category API, AMS 5]

FormalConjectures/Wikipedia/PebblingNumberConjecture.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -93,7 +93,7 @@ The pebbling number of the complete graph on `n` vertices is `n`.
9393
-/
9494
@[category API, AMS 5]
9595
theorem PebblingNumber_completeGraph [Fintype V] :
96-
PebblingNumber (completeGraph V) = Fintype.card V := by
96+
PebblingNumber (SimpleGraph.completeGraph V) = Fintype.card V := by
9797
refine IsLeast.csInf_eq ⟨fun D hD v => ?_, fun a ha => not_lt.1 fun ha_lt => ?_⟩
9898
· by_cases h : ∃ w, 2 ≤ D w
9999
· obtain ⟨w, hw⟩ := h

FormalConjectures/Wikipedia/RegularPrimes.lean

Lines changed: 1 addition & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -32,15 +32,10 @@ noncomputable section
3232

3333
variable (p : ℕ)
3434

35-
/-- TODO: remove this once mathlib is updated as it seems that in this version of mathlib
36-
we need to do this manually. -/
37-
instance [hp : Fact p.Prime] : NumberField (CyclotomicField ⟨p, hp.out.pos⟩ ℚ) :=
38-
IsCyclotomicExtension.numberField {⟨p, hp.out.pos⟩} ℚ _
39-
4035
/-- A natural prime number `p` is regular if `p` is coprime with the order of the class group
4136
of the `p`-th cyclotomic field. -/
4237
def IsRegularPrime [hp : Fact p.Prime] : Prop :=
43-
p.Coprime <| Fintype.card <| ClassGroup (𝓞 <| CyclotomicField ⟨p, hp.out.pos⟩ ℚ)
38+
p.Coprime <| Fintype.card <| ClassGroup (𝓞 <| CyclotomicField p ℚ)
4439

4540
@[category undergraduate, AMS 11]
4641
example : ¬ @IsRegularPrime 37 (by decide) := by

FormalConjectures/Wikipedia/UnionClosed.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -155,7 +155,7 @@ theorem union_closed.variants.sharpness [Fintype n] (c : ℝ) (hc : 1 / 2 < c) :
155155
obtain hn | hn := isEmpty_or_nonempty n
156156
· specialize h ∅
157157
simp only [ne_eq, card_empty, CharP.cast_eq_zero, mul_zero, filter_empty, le_refl,
158-
IsEmpty.exists_iff, imp_false, not_forall, not_mem_empty, imp_self, implies_true,
158+
IsEmpty.exists_iff, imp_false, not_forall, notMem_empty, imp_self, implies_true,
159159
not_true_eq_false, exists_const, Decidable.not_not] at h
160160
have : ∅ ∈ (∅ : Finset (Finset n)) := by simp [h]
161161
simp at this

docbuild/lakefile.toml

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -7,11 +7,11 @@ packagesDir = "../.lake/packages"
77
name = "formal_conjectures"
88
path = "../"
99

10-
# using fork here, because it contains a backported fix. Can be dropped after bump to v4.20.0
1110
[[require]]
1211
name = "doc-gen4"
13-
git = "https://github.com/mo271/doc-gen4"
14-
rev = "b760b91540bcf92c2ab6ac2bc28207e090769da8"
12+
scope = "leanprover"
13+
name = "doc-gen4"
14+
rev = "v4.20.1"
1515

1616
[[lean_exe]]
1717
name = "overwrite_index"

lake-manifest.json

Lines changed: 11 additions & 11 deletions
Original file line numberDiff line numberDiff line change
@@ -5,17 +5,17 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "leanprover-community",
8-
"rev": "c44e0c8ee63ca166450922a373c7409c5d26b00b",
8+
"rev": "5c0c94b3f563ed756b48b9439788c53b0d56a897",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
11-
"inputRev": "v4.19.0",
11+
"inputRev": "v4.20.1",
1212
"inherited": false,
1313
"configFile": "lakefile.lean"},
1414
{"url": "https://github.com/leanprover-community/plausible",
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "leanprover-community",
18-
"rev": "77e08eddc486491d7b9e470926b3dbe50319451a",
18+
"rev": "2ac43674e92a695e96caac19f4002b25434636da",
1919
"name": "plausible",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "main",
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "25078369972d295301f5a1e53c3e5850cf6d9d4c",
28+
"rev": "6c62474116f525d2814f0157bb468bf3a4f9f120",
2929
"name": "LeanSearchClient",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "main",
@@ -35,7 +35,7 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "e6a9f0f5ee3ccf7443a0070f92b62f8db12ae82b",
38+
"rev": "a11bcb5238149ae5d8a0aa5e2f8eddf8a3a9b27d",
3939
"name": "importGraph",
4040
"manifestFile": "lake-manifest.json",
4141
"inputRev": "main",
@@ -45,17 +45,17 @@
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "c4919189477c3221e6a204008998b0d724f49904",
48+
"rev": "21e6a0522cd2ae6cf88e9da99a1dd010408ab306",
4949
"name": "proofwidgets",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "v0.0.57",
51+
"inputRev": "v0.0.60",
5252
"inherited": true,
5353
"configFile": "lakefile.lean"},
5454
{"url": "https://github.com/leanprover-community/aesop",
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "5d50b08dedd7d69b3d9b3176e0d58a23af228884",
58+
"rev": "ddfca7829bf8aa4083cdf9633935dddbb28b7b2a",
5959
"name": "aesop",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "master",
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "fa4f7f15d97591a9cf3aa7724ba371c7fc6dda02",
68+
"rev": "2865ea099ab1dd8d6fc93381d77a4ac87a85527a",
6969
"name": "Qq",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "master",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "f5d04a9c4973d401c8c92500711518f7c656f034",
78+
"rev": "7a0d63fbf8fd350e891868a06d9927efa545ac1e",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",
@@ -85,7 +85,7 @@
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover",
88-
"rev": "02dbd02bc00ec4916e99b04b2245b30200e200d0",
88+
"rev": "f9e25dcbed001489c53bceeb1f1d50bbaf7451d4",
8989
"name": "Cli",
9090
"manifestFile": "lake-manifest.json",
9191
"inputRev": "main",

0 commit comments

Comments
 (0)