Skip to content

Commit

Permalink
refactor
Browse files Browse the repository at this point in the history
  • Loading branch information
iehality committed Sep 14, 2024
1 parent 77c9fbb commit 622ebb7
Show file tree
Hide file tree
Showing 2 changed files with 13 additions and 4 deletions.
3 changes: 2 additions & 1 deletion Incompleteness/Arith/First.lean
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,8 @@ lemma re_iff_sigma1 {P : ℕ → Prop} : RePred P ↔ 𝚺₁-Predicate P := by

variable (T : Theory ℒₒᵣ) [𝐑₀ ≼ T] [Sigma1Sound T] [T.Delta1Definable]

theorem incomplete : ¬System.Complete T := by
/-- Gödel's First Incompleteness Theorem-/
theorem goedel_first_incompleteness : ¬System.Complete T := by
let D : ℕ → Prop := fun n : ℕ ↦ ∃ p : SyntacticSemiformula ℒₒᵣ 1, n = ⌜p⌝ ∧ T ⊢! ∼p/[⌜p⌝]
have D_re : RePred D := by
have : 𝚺₁-Predicate fun p : ℕ ↦
Expand Down
14 changes: 11 additions & 3 deletions Incompleteness/Arith/Second.lean
Original file line number Diff line number Diff line change
Expand Up @@ -138,6 +138,8 @@ end

section

variable (T)

variable [T.Delta1Definable]

open LO.System LO.System.FiniteContext
Expand Down Expand Up @@ -179,11 +181,17 @@ lemma consistent_iff_goedel : T ⊢! ↑𝗖𝗼𝗻 ⭤ ↑𝗚 := by
simpa [provable₀_iff] using contra₁'! (deduct'! this)

/-- Gödel's Second Incompleteness Theorem-/
theorem consistent_unprovable [System.Consistent T] : T ⊬ ↑𝗖𝗼𝗻 := fun h ↦
goedel_unprovable <| and_left! consistent_iff_goedel ⨀ h
theorem goedel_second_incompleteness [System.Consistent T] : T ⊬ ↑𝗖𝗼𝗻 := fun h ↦
goedel_unprovable T <| and_left! (consistent_iff_goedel T) ⨀ h

theorem inconsistent_unprovable [ℕ ⊧ₘ* T] : T ⊬ ∼↑𝗖𝗼𝗻 := fun h ↦
not_goedel_unprovable <| contra₀'! (and_right! (consistent_iff_goedel (T := T))) ⨀ h
not_goedel_unprovable T <| contra₀'! (and_right! (consistent_iff_goedel T)) ⨀ h

theorem inconsistent_undecidable [ℕ ⊧ₘ* T] : System.Undecidable T ↑𝗖𝗼𝗻 := by
haveI : Consistent T := Sound.consistent_of_satisfiable ⟨_, (inferInstance : ℕ ⊧ₘ* T)⟩
constructor
· exact goedel_second_incompleteness T
· exact inconsistent_unprovable T

end

Expand Down

0 comments on commit 622ebb7

Please sign in to comment.