Change the literal type in a Clause
from α
to β
by using r
.
Equations
- Std.Sat.CNF.Clause.relabel r c = List.map (fun (x : Std.Sat.Literal α) => match x with | (i, n) => (r i, n)) c
Instances For
Relabelling #
It is convenient to be able to construct a CNF using a more complicated literal type,
but eventually we need to embed in Nat
.
Change the literal type in a CNF
formula from α
to β
by using r
.
Equations
Instances For
theorem
Std.Sat.CNF.nonempty_or_impossible
{α : Type u_1}
(f : CNF α)
:
Nonempty α ∨ ∃ (n : Nat), f = List.replicate n []