Skip to content

Commit

Permalink
sorry-free Bml.Completeness
Browse files Browse the repository at this point in the history
  • Loading branch information
m4lvin committed Oct 30, 2023
1 parent 53df4cc commit b24c248
Showing 1 changed file with 11 additions and 24 deletions.
35 changes: 11 additions & 24 deletions Bml/Completeness.lean
Original file line number Diff line number Diff line change
Expand Up @@ -158,35 +158,22 @@ theorem locTabEndSatThenSat {X Y} (ltX : LocalTableau X) (Y_endOf_X : Y ∈ endN
subst W_def
exact Y_endOf_W
case nCo ϕ ψ _ =>
simp at *
rw [nCoEndNodes, Finset.mem_union] at Y_endOf_X
cases Y_endOf_X
case inl Y_endOf_X =>
left
simp at *
sorry
/-
rcases Y_endOf_X with ⟨W, W_def, Y_endOf_W⟩
subst W_def
specialize IH (insert (~ϕ) (X.erase (~(ϕ⋀ψ))))
simp at IH
use insert (~ϕ) (X.erase (~(ϕ⋀ψ)))
specialize IH (X \ {~(ϕ⋀ψ)} ∪ {~ϕ})
use X \ {~(ϕ⋀ψ)} ∪ {~ϕ}
constructor
· left; rfl
· apply IH; exact Y_endOf_W
-/
· simp
· apply IH
convert Y_endOf_X;
case inr Y_endOf_X =>
right
sorry
/-
rcases Y_endOf_X with ⟨W, W_def, Y_endOf_W⟩
subst W_def
specialize IH (insert (~ψ) (X.erase (~(ϕ⋀ψ))))
simp at IH
use insert (~ψ) (X.erase (~(ϕ⋀ψ)))
specialize IH (X \ {~(ϕ⋀ψ)} ∪ {~ψ})
use X \ {~(ϕ⋀ψ)} ∪ {~ψ}
constructor
· right; rfl
· apply IH; exact Y_endOf_W
-/
· simp
· apply IH
convert Y_endOf_X;
case sim X simpX => aesop

theorem almostCompleteness : ∀ n X, lengthOfSet X = n → Consistent X → Satisfiable X :=
Expand Down

0 comments on commit b24c248

Please sign in to comment.