Skip to content
This repository was archived by the owner on Mar 8, 2025. It is now read-only.

Commit 92025de

Browse files
committed
update
1 parent 20f1429 commit 92025de

File tree

4 files changed

+20
-20
lines changed

4 files changed

+20
-20
lines changed

Incompleteness/Arith/FormalizedArithmetic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -250,7 +250,7 @@ noncomputable def nltNumeral (t : ⌜ℒₒᵣ⌝.Term) (n : V) : T ⊢ t ≮'
250250
def ltComplete {n m : V} (h : n < m) : T ⊢ ↑n <' ↑m := by
251251
have : T ⊢ ↑n <' ↑m ⭤ _ := ltNumeral T n m
252252
apply andRight this ⨀ ?_
253-
apply disj (i := m - (n + 1)) _ (by simpa using sub_succ_lt_self (by simp [h]))
253+
apply disj (i := m - (n + 1)) _ (by simpa using sub_succ_lt_self h)
254254
simpa [nth_tSubstItr', h] using eqRefl T ↑n
255255

256256
lemma lt_complete! {n m : V} (h : n < m) : T ⊢! ↑n <' ↑m := ⟨ltComplete T h⟩

Incompleteness/Arith/Second.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -18,7 +18,7 @@ lemma substNumeral_app_quote (σ : Semisentence ℒₒᵣ 1) (n : ℕ) :
1818
substNumeral ⌜σ⌝ (n : V) = ⌜(σ/[‘↑n’] : Sentence ℒₒᵣ)⌝ := by
1919
dsimp [substNumeral]
2020
let w : Fin 1 → Semiterm ℒₒᵣ Empty 0 := ![‘↑n’]
21-
have : ?[numeral (n : V)] = (⌜fun i : Fin 1 ↦ ⌜w i⌝⌝ : V) := nth_ext' 1 (by simp) (by simp) (by simp)
21+
have : ?[numeral (n : V)] = (⌜fun i : Fin 1 ↦ ⌜w i⌝⌝ : V) := nth_ext' 1 (by simp) (by simp) (by simp [w])
2222
rw [Language.substs₁, this, quote_substs' (L := ℒₒᵣ)]
2323

2424
lemma substNumeral_app_quote_quote (σ π : Semisentence ℒₒᵣ 1) :
@@ -108,7 +108,7 @@ theorem diagonal (θ : Semisentence ℒₒᵣ 1) :
108108
let Θ : V → Prop := fun x ↦ Semiformula.Evalbm V ![x] θ
109109
calc
110110
V ⊧/![] (fixpoint θ)
111-
↔ Θ (substNumeral ⌜diag θ⌝ ⌜diag θ⌝) := by simp [fixpoint_eq]
111+
↔ Θ (substNumeral ⌜diag θ⌝ ⌜diag θ⌝) := by simp [Θ, fixpoint_eq]
112112
_ ↔ Θ ⌜fixpoint θ⌝ := by simp [substNumeral_app_quote_quote]; rfl
113113

114114
end Diagonalization
@@ -133,7 +133,7 @@ theorem multidiagonal (θ : Fin k → Semisentence ℒₒᵣ k) :
133133
have ht : ∀ i, substNumerals (t i) t = ⌜multifixpoint θ i⌝ := by
134134
intro i; simp [t, multifixpoint, substNumerals_app_quote_quote]
135135
calc
136-
V ⊧/![] (multifixpoint θ i) ↔ V ⊧/t (multidiag (θ i)) := by simp [multifixpoint]
136+
V ⊧/![] (multifixpoint θ i) ↔ V ⊧/t (multidiag (θ i)) := by simp [t, multifixpoint]
137137
_ ↔ V ⊧/(fun i ↦ substNumerals (t i) t) (θ i) := by simp [multidiag, ← funext_iff]
138138
_ ↔ V ⊧/(fun i ↦ ⌜multifixpoint θ i⌝) (θ i) := by simp [ht]
139139

lake-manifest.json

Lines changed: 15 additions & 15 deletions
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "FormalizedFormalLogic",
8-
"rev": "f820bd432d95be117b857b9a00823b1de395fd88",
8+
"rev": "d3e3fb955304f6f5c97abfac96f0e30e18b74f05",
99
"name": "arithmetization",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": "master",
@@ -15,7 +15,7 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "FormalizedFormalLogic",
18-
"rev": "0325e10aefcc4025554b4c188d268cd3d830ba21",
18+
"rev": "54324e6e009f0d0a288897312d3feb1c0165ad19",
1919
"name": "foundation",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "master",
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "e423a1f0105a779265101af2bd177f5d8065c594",
28+
"rev": "8fac96b567d5b979e6a55c99158a99b20e968a96",
2929
"name": "mathlib",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "master",
@@ -35,10 +35,10 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "8e5cb8d424df462f84997dd68af6f40e347c3e35",
38+
"rev": "1622a8693b31523c8f82db48e01b14c74bc1f155",
3939
"name": "plausible",
4040
"manifestFile": "lake-manifest.json",
41-
"inputRev": "v4.15.0-rc1",
41+
"inputRev": "v4.16.0-rc1",
4242
"inherited": true,
4343
"configFile": "lakefile.toml"},
4444
{"url": "https://github.com/leanprover-community/LeanSearchClient",
@@ -55,47 +55,47 @@
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "ed3b856bd8893ade75cafe13e8544d4c2660f377",
58+
"rev": "f72319c9686788305a8ab059f3c4d8c724785c83",
5959
"name": "importGraph",
6060
"manifestFile": "lake-manifest.json",
61-
"inputRev": "v4.15.0-rc1",
61+
"inputRev": "main",
6262
"inherited": true,
6363
"configFile": "lakefile.toml"},
6464
{"url": "https://github.com/leanprover-community/ProofWidgets4",
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "2b000e02d50394af68cfb4770a291113d94801b5",
68+
"rev": "07f60e90998dfd6592688a14cd67bd4e384b77b2",
6969
"name": "proofwidgets",
7070
"manifestFile": "lake-manifest.json",
71-
"inputRev": "v0.0.48",
71+
"inputRev": "v0.0.50",
7272
"inherited": true,
7373
"configFile": "lakefile.lean"},
7474
{"url": "https://github.com/leanprover-community/aesop",
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "a4a08d92be3de00def5298059bf707c72dfd3c66",
78+
"rev": "79402ad9ab4be9a2286701a9880697e2351e4955",
7979
"name": "aesop",
8080
"manifestFile": "lake-manifest.json",
81-
"inputRev": "master",
81+
"inputRev": "v4.16.0-rc1",
8282
"inherited": true,
8383
"configFile": "lakefile.toml"},
8484
{"url": "https://github.com/leanprover-community/quote4",
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover-community",
88-
"rev": "ad942fdf0b15c38bface6acbb01d63855a2519ac",
88+
"rev": "f0c584bcb14c5adfb53079781eeea75b26ebbd32",
8989
"name": "Qq",
9090
"manifestFile": "lake-manifest.json",
91-
"inputRev": "v4.14.0",
91+
"inputRev": "v4.15.0",
9292
"inherited": true,
93-
"configFile": "lakefile.lean"},
93+
"configFile": "lakefile.toml"},
9494
{"url": "https://github.com/leanprover-community/batteries",
9595
"type": "git",
9696
"subDir": null,
9797
"scope": "leanprover-community",
98-
"rev": "f007bfe46ea8fb801ec907df9ab540054abcc5fd",
98+
"rev": "5b23a1297aba9683f231c4b1a7ab4076af4ad53d",
9999
"name": "batteries",
100100
"manifestFile": "lake-manifest.json",
101101
"inputRev": "main",

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.15.0-rc1
1+
leanprover/lean4:v4.16.0-rc2

0 commit comments

Comments
 (0)