Skip to content

Commit

Permalink
fix(FirstOrder): Sigma1Sound
Browse files Browse the repository at this point in the history
  • Loading branch information
iehality committed Dec 12, 2024
1 parent cca37b3 commit 9033902
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions Foundation/FirstOrder/Arith/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -184,15 +184,15 @@ end BinderNotation
namespace Arith

class SoundOn {L : Language} [Structure L ℕ]
(T : Theory L) (F : SyntacticFormula L → Prop) where
sound : ∀ {φ}, F φ → T ⊢! φ → ℕ ⊧ₘ φ
(T : Theory L) (F : Sentence L → Prop) where
sound : ∀ {σ}, F σ → T ⊢! ↑σ → ℕ ⊧ₘ₀ σ

section

variable {L : Language} [Structure L ℕ] (T : Theory L) (F : Set (SyntacticFormula L))
variable {L : Language} [Structure L ℕ] (T : Theory L) (F : Set (Sentence L))

lemma consistent_of_sound [SoundOn T F] (hF : ⊥ ∈ F) : System.Consistent T :=
System.consistent_iff_unprovable_bot.mpr fun b ↦ by simpa using SoundOn.sound (F := F) hF b
System.consistent_iff_unprovable_bot.mpr fun b ↦ by simpa [Models₀] using SoundOn.sound (F := F) hF b

end

Expand Down

0 comments on commit 9033902

Please sign in to comment.