src/Tools/Metis/src/Problem.sig
changeset 39347 50dec19e682b
parent 39346 d837998f1e60
child 39348 6f9c9899f99f
--- a/src/Tools/Metis/src/Problem.sig	Mon Sep 13 20:27:40 2010 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,57 +0,0 @@
-(* ========================================================================= *)
-(* SOME SAMPLE PROBLEMS TO TEST PROOF PROCEDURES                             *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
-(* ========================================================================= *)
-
-signature Problem =
-sig
-
-(* ------------------------------------------------------------------------- *)
-(* Problems.                                                                 *)
-(* ------------------------------------------------------------------------- *)
-
-type problem = Thm.clause list
-
-val size : problem -> {clauses : int,
-                       literals : int,
-                       symbols : int,
-                       typedSymbols : int}
-
-val fromGoal : Formula.formula -> problem list
-
-val toClauses : problem -> Formula.formula
-
-val toString : problem -> string
-
-(* ------------------------------------------------------------------------- *)
-(* Categorizing problems.                                                    *)
-(* ------------------------------------------------------------------------- *)
-
-datatype propositional =
-    Propositional
-  | EffectivelyPropositional
-  | NonPropositional
-
-datatype equality =
-    NonEquality
-  | Equality
-  | PureEquality
-
-datatype horn =
-    Trivial
-  | Unit
-  | DoubleHorn
-  | Horn
-  | NegativeHorn
-  | NonHorn
-
-type category =
-     {propositional : propositional,
-      equality : equality,
-      horn : horn}
-
-val categorize : problem -> category
-
-val categoryToString : category -> string
-
-end