Skip to content

Commit

Permalink
fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
fpvandoorn authored and PatrickMassot committed Feb 19, 2025
1 parent 4c929fb commit 69e817b
Show file tree
Hide file tree
Showing 2 changed files with 6 additions and 6 deletions.
Original file line number Diff line number Diff line change
Expand Up @@ -55,17 +55,17 @@ def Valid (A : Formula) : Prop := ∅ ⊨ A
using theorems tagged with `@[simp]`. -/

variable {v : Variable → Prop} {A B : Formula}
@[simp] lemma isTrue_neg : IsTrue v ~A ↔ ¬ IsTrue v A := by simp
@[simp] lemma isTrue_neg : IsTrue v ~A ↔ ¬ IsTrue v A := by simp [neg]

@[simp] lemma isTrue_top : IsTrue v ⊤ := by {
-- sorry
simp
simp [top]
-- sorry
}

@[simp] lemma isTrue_equiv : IsTrue v (A ⇔ B) ↔ (IsTrue v A ↔ IsTrue v B) := by {
-- sorry
simp
simp [equiv]
tauto
-- sorry
}
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -62,18 +62,18 @@ def Valid (A : Formula) : Prop := ∅ ⊨ A
using theorems tagged with `@[simp]`. -/

variable {v : Variable → H} {A B : Formula}
@[simp] lemma eval_neg : eval v ~A = (eval v A)ᶜ := by simp
@[simp] lemma eval_neg : eval v ~A = (eval v A)ᶜ := by simp [neg]

@[simp] lemma eval_top : eval v top = ⊤ := by {
-- sorry
simp
simp [top]
-- sorry
}

@[simp]
lemma isTrue_equiv : eval v (A ⇔ B) = (eval v A ⇨ eval v B) ⊓ (eval v B ⇨ eval v A) := by {
-- sorry
simp
simp [equiv]
-- sorry
}

Expand Down

0 comments on commit 69e817b

Please sign in to comment.