Skip to content

Commit

Permalink
wkFmlLₕ
Browse files Browse the repository at this point in the history
  • Loading branch information
SnO2WMaN committed Dec 17, 2024
1 parent 691b0fb commit 32a27cb
Show file tree
Hide file tree
Showing 6 changed files with 434 additions and 319 deletions.
11 changes: 7 additions & 4 deletions LabelledSystem/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,9 @@ namespace Labelled

abbrev Label := ℕ

abbrev PropVar := ℕ


def Assignment (M : Kripke.Model) := Label → M.World


Expand Down Expand Up @@ -70,7 +73,7 @@ end LabelTerm

structure LabelledFormula where
label : Label
formula : Formula
formula : Formula PropVar
deriving DecidableEq, Repr

namespace LabelledFormula
Expand All @@ -83,7 +86,7 @@ notation lφ "⟦" σ "⟧" => labelReplace σ lφ

section

variable {x y z : Label} {φ ψ : Formula } {σ : LabelReplace}
variable {x y z : Label} {φ ψ : Formula PropVar} {σ : LabelReplace}

@[simp]
lemma def_labelReplace : (x ∶ φ).labelReplace σ = (σ x ∶ φ) := by rfl
Expand All @@ -106,7 +109,7 @@ protected instance semantics {M : Kripke.Model} : Semantics (LabelledFormula) (A

variable {M : Kripke.Model} {f : Assignment M}
variable {x y : Label}
variable {φ ψ : Formula } {xφ: LabelledFormula}
variable {φ ψ : Formula PropVar} {xφ: LabelledFormula}

@[simp] protected lemma iff_models : f ⊧ (x ∶ φ) ↔ f x ⊧ φ := by tauto;

Expand All @@ -121,7 +124,7 @@ end LabelledFormula

structure LabelledNNFormula where
label : Label
formula : NNFormula
formula : NNFormula PropVar
deriving DecidableEq, Repr

end Labelled
Expand Down
Loading

0 comments on commit 32a27cb

Please sign in to comment.