File tree Expand file tree Collapse file tree 2 files changed +2
-3
lines changed Expand file tree Collapse file tree 2 files changed +2
-3
lines changed Original file line number Diff line number Diff line change @@ -53,7 +53,7 @@ theorem sat_def (a : α → Bool) (f : CNF α) : Sat a f ↔ (eval a f = true) :
53
53
theorem unsat_def (f : CNF α) : Unsat f ↔ (∀ a, eval a f = false ) := by rfl
54
54
55
55
56
- @[simp] theorem not_unsatisfiable_nil : ¬Unsat ([] : CNF α) :=
56
+ @[simp] theorem not_unsat_nil : ¬Unsat ([] : CNF α) :=
57
57
fun h => by simp [unsat_def] at h
58
58
59
59
@[simp] theorem sat_nil {assign : α → Bool} : Sat assign ([] : CNF α) := by
Original file line number Diff line number Diff line change @@ -113,8 +113,7 @@ def relabelFin (f : CNF Nat) : CNF (Fin f.numLiterals) :=
113
113
else
114
114
List.replicate f.length []
115
115
116
- theorem unsat_relabelFin {f : CNF Nat} :
117
- Unsat f.relabelFin ↔ Unsat f := by
116
+ @[simp] theorem unsat_relabelFin {f : CNF Nat} : Unsat f.relabelFin ↔ Unsat f := by
118
117
dsimp [relabelFin]
119
118
split <;> rename_i h
120
119
· apply unsat_relabel_iff
You can’t perform that action at this time.
0 commit comments