src/Tools/Metis/src/Normalize.sig
author haftmann
Mon, 16 Feb 2009 19:11:55 +0100
changeset 29940 83b373f61d41
parent 23510 4521fead5609
child 39353 7f11d833d65b
permissions -rw-r--r--
more default simp rules for sgn

(* ========================================================================= *)
(* NORMALIZING FORMULAS                                                      *)
(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
(* ========================================================================= *)

signature Normalize =
sig

(* ------------------------------------------------------------------------- *)
(* Negation normal form.                                                     *)
(* ------------------------------------------------------------------------- *)

val nnf : Formula.formula -> Formula.formula

(* ------------------------------------------------------------------------- *)
(* Conjunctive normal form.                                                  *)
(* ------------------------------------------------------------------------- *)

val cnf : Formula.formula -> Formula.formula list

end