Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
SnO2WMaN committed Dec 6, 2024
1 parent d30eb5b commit 4844617
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 4 deletions.
1 change: 1 addition & 0 deletions LabelledSystem.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,3 +2,4 @@ import LabelledSystem.Basic

import LabelledSystem.Gentzen.Basic
import LabelledSystem.Gentzen.Soundness
import LabelledSystem.Gentzen.Hilbert
4 changes: 2 additions & 2 deletions LabelledSystem/Gentzen/Hilbert.lean
Original file line number Diff line number Diff line change
Expand Up @@ -56,8 +56,8 @@ def axiomK : ⊢ᵍ ⟨∅, ∅⟩ ⟹ ⟨{x ∶ □(φ ➝ ψ) ➝ □φ ➝
have e : (x ∶ □(φ ➝ ψ)) ::ₘ (y ∶ φ ➝ ψ) ::ₘ (y ∶ φ) ::ₘ {x ∶ □φ} = (y ∶ φ ➝ ψ) ::ₘ {y ∶ φ, x ∶ □φ, x ∶ □(φ ➝ ψ)} := by sorry;
simpa [e];
apply impL (Γ := ⟨_, _⟩);
. simpa using initFml (Γ := ⟨_, _⟩) (Δ := ⟨_, _⟩);
. simpa using initFml (Γ := ⟨_, _⟩) (Δ := ⟨_, _⟩);
. exact initFml' y φ (by simp) (by simp);
. exact initFml' y ψ (by simp) (by simp);

def mdp (d₁ : ⊢ᵍ ⟨∅, ∅⟩ ⟹ ⟨{x ∶ φ ➝ ψ}, ∅⟩) (d₂ : ⊢ᵍ ⟨∅, ∅⟩ ⟹ ⟨{x ∶ φ}, ∅⟩) : ⊢ᵍ ⟨∅, ∅⟩ ⟹ ⟨{x ∶ ψ}, ∅⟩ := by
simpa using cutFml (Δ₁ := ⟨∅, ∅⟩) (Δ₂ := ⟨{x ∶ ψ}, ∅⟩) d₂ $ implyRInv (Δ := ⟨∅, ∅⟩) d₁;
Expand Down
4 changes: 2 additions & 2 deletions LabelledSystem/Gentzen/Soundness.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,10 +5,10 @@ namespace LO.Modal.Labelled.Gentzen
theorem soundness {S : Sequent} : ⊢ᵍ S → ∀ (M : Kripke.Model), ∀ (f : Assignment M), S.Satisfies M f := by
intro d;
induction d with
| axA =>
| initAtom =>
rintro M f ⟨hΓ, hX⟩;
simp_all;
| axBot =>
| initBot =>
rintro M f ⟨hΓ, hX⟩;
simp at hΓ;
| @impL Γ Δ x φ ψ d₁ d₂ ih₁ ih₂ =>
Expand Down

0 comments on commit 4844617

Please sign in to comment.