Skip to content

Commit

Permalink
add small notes
Browse files Browse the repository at this point in the history
  • Loading branch information
m4lvin committed Dec 17, 2023
1 parent a565ac2 commit 5d797ea
Showing 1 changed file with 5 additions and 4 deletions.
9 changes: 5 additions & 4 deletions Pdl/DagTableau.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,8 +8,8 @@ import Pdl.Star
import Pdl.Closure

inductive DagFormula : Type
| dag : Program → Formula → DagFormula
| box : Program → DagFormula → DagFormula
| dag : Program → Formula → DagFormula -- ⌈a†⌉f
| box : Program → DagFormula → DagFormula -- ⌈a⌉df
deriving Repr, DecidableEq

@[simp]
Expand Down Expand Up @@ -332,15 +332,15 @@ decreasing_by simp_wf; assumption

theorem dagEnd_subset_next :
Ω ∈ dagNext Γ → dagEndNodes Ω ⊆ dagEndNodes Γ := by
sorry
sorry -- medium?

-- A normal successor is an endNode.
theorem dagNormal_is_dagEnd
(Γ_in : Γ ∈ dagNextTransRefl S)
(Γ_normal : Γ.2 = none)
:
(Γ.1 ∈ dagEndNodes S) := by
sorry
sorry -- should be easy

theorem dagEnd_subset_trf {Ω Γ} :
Ω ∈ dagNextTransRefl Γ → dagEndNodes Ω ⊆ dagEndNodes Γ := by
Expand Down Expand Up @@ -420,3 +420,4 @@ decreasing_by simp_wf; assumption
theorem starSoundness (M : KripkeModel W) (v : W) :
(M, v) ⊨ S ↔ ∃ Γ ∈ boxDagEndNodes S, (M, v) ⊨ Γ := by
sorry
-- TODO: this is not true, needs to be adjusted or done in Tableau.localRuleTruth dircetly, like in the diamond case.

0 comments on commit 5d797ea

Please sign in to comment.