GPL -> BSD
authorpaulson
Wed, 27 Jun 2007 12:41:36 +0200
changeset 23510 4521fead5609
parent 23509 14a2f87ccc73
child 23511 7067f5e3670f
GPL -> BSD
src/Tools/Metis/metis.ML
src/Tools/Metis/src/Active.sig
src/Tools/Metis/src/Active.sml
src/Tools/Metis/src/Atom.sig
src/Tools/Metis/src/Atom.sml
src/Tools/Metis/src/AtomNet.sig
src/Tools/Metis/src/AtomNet.sml
src/Tools/Metis/src/Clause.sig
src/Tools/Metis/src/Clause.sml
src/Tools/Metis/src/ElementSet.sig
src/Tools/Metis/src/ElementSet.sml
src/Tools/Metis/src/Formula.sig
src/Tools/Metis/src/Formula.sml
src/Tools/Metis/src/Heap.sig
src/Tools/Metis/src/Heap.sml
src/Tools/Metis/src/KeyMap.sig
src/Tools/Metis/src/KeyMap.sml
src/Tools/Metis/src/KnuthBendixOrder.sig
src/Tools/Metis/src/KnuthBendixOrder.sml
src/Tools/Metis/src/Lazy.sig
src/Tools/Metis/src/Lazy.sml
src/Tools/Metis/src/Literal.sig
src/Tools/Metis/src/Literal.sml
src/Tools/Metis/src/LiteralNet.sig
src/Tools/Metis/src/LiteralNet.sml
src/Tools/Metis/src/Map.sig
src/Tools/Metis/src/Map.sml
src/Tools/Metis/src/Model.sig
src/Tools/Metis/src/Model.sml
src/Tools/Metis/src/Name.sig
src/Tools/Metis/src/Name.sml
src/Tools/Metis/src/Normalize.sig
src/Tools/Metis/src/Normalize.sml
src/Tools/Metis/src/Options.sig
src/Tools/Metis/src/Options.sml
src/Tools/Metis/src/Ordered.sig
src/Tools/Metis/src/Ordered.sml
src/Tools/Metis/src/Parser.sig
src/Tools/Metis/src/Parser.sml
src/Tools/Metis/src/Portable.sig
src/Tools/Metis/src/PortableMlton.sml
src/Tools/Metis/src/PortableMosml.sml
src/Tools/Metis/src/PortableSmlNJ.sml
src/Tools/Metis/src/Problem.sig
src/Tools/Metis/src/Problem.sml
src/Tools/Metis/src/Proof.sig
src/Tools/Metis/src/Proof.sml
src/Tools/Metis/src/RandomMap.sml
src/Tools/Metis/src/RandomSet.sml
src/Tools/Metis/src/Resolution.sig
src/Tools/Metis/src/Resolution.sml
src/Tools/Metis/src/Rewrite.sig
src/Tools/Metis/src/Rewrite.sml
src/Tools/Metis/src/Rule.sig
src/Tools/Metis/src/Rule.sml
src/Tools/Metis/src/Set.sig
src/Tools/Metis/src/Set.sml
src/Tools/Metis/src/Sharing.sig
src/Tools/Metis/src/Sharing.sml
src/Tools/Metis/src/Stream.sig
src/Tools/Metis/src/Stream.sml
src/Tools/Metis/src/Subst.sig
src/Tools/Metis/src/Subst.sml
src/Tools/Metis/src/Subsume.sig
src/Tools/Metis/src/Subsume.sml
src/Tools/Metis/src/Term.sig
src/Tools/Metis/src/Term.sml
src/Tools/Metis/src/TermNet.sig
src/Tools/Metis/src/TermNet.sml
src/Tools/Metis/src/Thm.sig
src/Tools/Metis/src/Thm.sml
src/Tools/Metis/src/Tptp.sig
src/Tools/Metis/src/Tptp.sml
src/Tools/Metis/src/Units.sig
src/Tools/Metis/src/Units.sml
src/Tools/Metis/src/Useful.sig
src/Tools/Metis/src/Useful.sml
src/Tools/Metis/src/Waiting.sig
src/Tools/Metis/src/Waiting.sml
src/Tools/Metis/src/problems.sml
src/Tools/Metis/src/problems2tptp.sml
--- a/src/Tools/Metis/metis.ML	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/metis.ML	Wed Jun 27 12:41:36 2007 +0200
@@ -13,7 +13,7 @@
 
 (* ========================================================================= *)
 (* ML SPECIFIC FUNCTIONS                                                     *)
-(* Copyright (c) 2001-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Portable =
@@ -1032,7 +1032,7 @@
 
 (* ========================================================================= *)
 (* ML UTILITY FUNCTIONS                                                      *)
-(* Copyright (c) 2001-2005 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2005 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Useful =
@@ -1345,7 +1345,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* ML UTILITY FUNCTIONS                                                      *)
-(* Copyright (c) 2001-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Useful :> Useful =
@@ -2040,7 +2040,7 @@
 
 (* ========================================================================= *)
 (* SUPPORT FOR LAZY EVALUATION                                               *)
-(* Copyright (c) 2007 Joe Hurd, distributed under the GNU GPL version 2      *)
+(* Copyright (c) 2007 Joe Hurd, distributed under the BSD License      *)
 (* ========================================================================= *)
 
 signature Lazy =
@@ -2066,7 +2066,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* SUPPORT FOR LAZY EVALUATION                                               *)
-(* Copyright (c) 2007 Joe Hurd, distributed under the GNU GPL version 2      *)
+(* Copyright (c) 2007 Joe Hurd, distributed under the BSD License      *)
 (* ========================================================================= *)
 
 structure Lazy :> Lazy =
@@ -2103,7 +2103,7 @@
 
 (* ========================================================================= *)
 (* ORDERED TYPES                                                             *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Ordered =
@@ -2145,7 +2145,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* ORDERED TYPES                                                             *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure IntOrdered =
@@ -2159,7 +2159,7 @@
 
 (* ========================================================================= *)
 (* FINITE SETS                                                               *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Set =
@@ -2281,7 +2281,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FINITE SETS IMPLEMENTED WITH RANDOMLY BALANCED TREES                      *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure RandomSet :> Set =
@@ -2898,7 +2898,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FINITE SETS                                                               *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Set = RandomSet;
@@ -2908,7 +2908,7 @@
 
 (* ========================================================================= *)
 (* FINITE SETS WITH A FIXED ELEMENT TYPE                                     *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature ElementSet =
@@ -3024,7 +3024,7 @@
 
 (* ========================================================================= *)
 (* FINITE SETS WITH A FIXED ELEMENT TYPE                                     *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 functor ElementSet (Key : Ordered) :> ElementSet where type element = Key.t =
@@ -3150,7 +3150,7 @@
 
 (* ========================================================================= *)
 (* FINITE MAPS                                                               *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Map =
@@ -3262,7 +3262,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FINITE MAPS IMPLEMENTED WITH RANDOMLY BALANCED TREES                      *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure RandomMap :> Map =
@@ -3893,7 +3893,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FINITE MAPS                                                               *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Map = RandomMap;
@@ -3903,7 +3903,7 @@
 
 (* ========================================================================= *)
 (* FINITE MAPS WITH A FIXED KEY TYPE                                         *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature KeyMap =
@@ -4009,7 +4009,7 @@
 
 (* ========================================================================= *)
 (* FINITE MAPS WITH A FIXED KEY TYPE                                         *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 functor KeyMap (Key : Ordered) :> KeyMap where type key = Key.t =
@@ -4127,7 +4127,7 @@
 
 (* ========================================================================= *)
 (* PRESERVING SHARING OF ML VALUES                                           *)
-(* Copyright (c) 2005-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2005-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Sharing =
@@ -4173,7 +4173,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* PRESERVING SHARING OF ML VALUES                                           *)
-(* Copyright (c) 2005-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2005-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Sharing :> Sharing =
@@ -4256,7 +4256,7 @@
 
 (* ========================================================================= *)
 (* A POSSIBLY-INFINITE STREAM DATATYPE FOR ML                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Stream =
@@ -4357,7 +4357,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* A POSSIBLY-INFINITE STREAM DATATYPE FOR ML                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Stream :> Stream =
@@ -4563,7 +4563,7 @@
 
 (* ========================================================================= *)
 (* A HEAP DATATYPE FOR ML                                                    *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Heap =
@@ -4603,7 +4603,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* A HEAP DATATYPE FOR ML                                                    *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Heap :> Heap =
@@ -4684,7 +4684,7 @@
 
 (* ========================================================================= *)
 (* PARSING AND PRETTY PRINTING                                               *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Parser =
@@ -4837,7 +4837,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* PARSER COMBINATORS                                                        *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Parser :> Parser =
@@ -5237,7 +5237,7 @@
 
 (* ========================================================================= *)
 (* PROCESSING COMMAND LINE OPTIONS                                           *)
-(* Copyright (c) 2003-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Options =
@@ -5339,7 +5339,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* PROCESSING COMMAND LINE OPTIONS                                           *)
-(* Copyright (c) 2003-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Options :> Options =
@@ -5597,7 +5597,7 @@
 
 (* ========================================================================= *)
 (* NAMES                                                                     *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Name =
@@ -5621,7 +5621,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* NAMES                                                                     *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Name :> Name =
@@ -5710,7 +5710,7 @@
 
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC TERMS                                                   *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Term =
@@ -5896,7 +5896,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC TERMS                                                   *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Term :> Term =
@@ -6560,7 +6560,7 @@
 
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC SUBSTITUTIONS                                           *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Subst =
@@ -6668,7 +6668,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC SUBSTITUTIONS                                           *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Subst :> Subst =
@@ -6880,7 +6880,7 @@
 
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC ATOMS                                                   *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Atom =
@@ -7026,7 +7026,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC ATOMS                                                   *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Atom :> Atom =
@@ -7275,7 +7275,7 @@
 
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC FORMULAS                                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Formula =
@@ -7463,7 +7463,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC FORMULAS                                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Formula :> Formula =
@@ -7982,7 +7982,7 @@
 
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC LITERALS                                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Literal =
@@ -8154,7 +8154,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC LITERALS                                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Literal :> Literal =
@@ -8431,7 +8431,7 @@
 
 (* ========================================================================= *)
 (* A LOGICAL KERNEL FOR FIRST ORDER CLAUSES                                  *)
-(* Copyright (c) 2001-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Thm =
@@ -8588,7 +8588,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* A LOGICAL KERNEL FOR FIRST ORDER CLAUSES                                  *)
-(* Copyright (c) 2001-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Thm :> Thm =
@@ -8815,7 +8815,7 @@
 
 (* ========================================================================= *)
 (* PROOFS IN FIRST ORDER LOGIC                                               *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Proof =
@@ -8873,7 +8873,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* PROOFS IN FIRST ORDER LOGIC                                               *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Proof :> Proof =
@@ -9256,7 +9256,7 @@
 
 (* ========================================================================= *)
 (* DERIVED RULES FOR CREATING FIRST ORDER LOGIC THEOREMS                     *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Rule =
@@ -9535,7 +9535,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* DERIVED RULES FOR CREATING FIRST ORDER LOGIC THEOREMS                     *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Rule :> Rule =
@@ -10302,7 +10302,7 @@
 
 (* ========================================================================= *)
 (* NORMALIZING FORMULAS                                                      *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Normalize =
@@ -10332,7 +10332,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* NORMALIZING FORMULAS                                                      *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Normalize :> Normalize =
@@ -11398,7 +11398,7 @@
 
 (* ========================================================================= *)
 (* RANDOM FINITE MODELS                                                      *)
-(* Copyright (c) 2003-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Model =
@@ -11501,7 +11501,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* RANDOM FINITE MODELS                                                      *)
-(* Copyright (c) 2003-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Model :> Model =
@@ -12104,7 +12104,7 @@
 
 (* ========================================================================= *)
 (* SOME SAMPLE PROBLEMS TO TEST PROOF PROCEDURES                             *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Problem =
@@ -12170,7 +12170,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* SOME SAMPLE PROBLEMS TO TEST PROOF PROCEDURES                             *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Problem :> Problem =
@@ -12359,7 +12359,7 @@
 
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC TERMS              *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature TermNet =
@@ -12418,7 +12418,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC TERMS              *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure TermNet :> TermNet =
@@ -12840,7 +12840,7 @@
 
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC ATOMS              *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature AtomNet =
@@ -12897,7 +12897,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC ATOMS              *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure AtomNet :> AtomNet =
@@ -12960,7 +12960,7 @@
 
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC LITERALS           *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature LiteralNet =
@@ -13019,7 +13019,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC LITERALS           *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure LiteralNet :> LiteralNet =
@@ -13097,7 +13097,7 @@
 
 (* ========================================================================= *)
 (* SUBSUMPTION CHECKING FOR FIRST ORDER LOGIC CLAUSES                        *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Subsume =
@@ -13157,7 +13157,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* SUBSUMPTION CHECKING FOR FIRST ORDER LOGIC CLAUSES                        *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Subsume :> Subsume =
@@ -13495,7 +13495,7 @@
 
 (* ========================================================================= *)
 (* THE KNUTH-BENDIX TERM ORDERING                                            *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature KnuthBendixOrder =
@@ -13526,7 +13526,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* KNUTH-BENDIX TERM ORDERING CONSTRAINTS                                    *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure KnuthBendixOrder :> KnuthBendixOrder =
@@ -13781,7 +13781,7 @@
 
 (* ========================================================================= *)
 (* ORDERED REWRITING FOR FIRST ORDER TERMS                                   *)
-(* Copyright (c) 2003-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Rewrite =
@@ -13877,7 +13877,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* ORDERED REWRITING FOR FIRST ORDER TERMS                                   *)
-(* Copyright (c) 2003-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Rewrite :> Rewrite =
@@ -14533,7 +14533,7 @@
 
 (* ========================================================================= *)
 (* A STORE FOR UNIT THEOREMS                                                 *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Units =
@@ -14591,7 +14591,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* A STORE FOR UNIT THEOREMS                                                 *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Units :> Units =
@@ -14701,7 +14701,7 @@
 
 (* ========================================================================= *)
 (* CLAUSE = ID + THEOREM                                                     *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Clause =
@@ -14815,7 +14815,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* CLAUSE = ID + THEOREM                                                     *)
-(* Copyright (c) 2002-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Clause :> Clause =
@@ -15168,7 +15168,7 @@
 
 (* ========================================================================= *)
 (* THE ACTIVE SET OF CLAUSES                                                 *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Active =
@@ -15227,7 +15227,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* THE ACTIVE SET OF CLAUSES                                                 *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Active :> Active =
@@ -16034,7 +16034,7 @@
 
 (* ========================================================================= *)
 (* THE WAITING SET OF CLAUSES                                                *)
-(* Copyright (c) 2002-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Waiting =
@@ -16091,7 +16091,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* THE WAITING SET OF CLAUSES                                                *)
-(* Copyright (c) 2002-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Waiting :> Waiting =
@@ -16272,7 +16272,7 @@
 
 (* ========================================================================= *)
 (* THE RESOLUTION PROOF PROCEDURE                                            *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Resolution =
@@ -16330,7 +16330,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* THE RESOLUTION PROOF PROCEDURE                                            *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Resolution :> Resolution =
@@ -16432,7 +16432,7 @@
 
 (* ========================================================================= *)
 (* INTERFACE TO TPTP PROBLEM FILES                                           *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Tptp =
@@ -16520,7 +16520,7 @@
 val print = TextIO.print;
 (* ========================================================================= *)
 (* INTERFACE TO TPTP PROBLEM FILES                                           *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Tptp :> Tptp =
--- a/src/Tools/Metis/src/Active.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Active.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* THE ACTIVE SET OF CLAUSES                                                 *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Active =
--- a/src/Tools/Metis/src/Active.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Active.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* THE ACTIVE SET OF CLAUSES                                                 *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Active :> Active =
--- a/src/Tools/Metis/src/Atom.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Atom.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC ATOMS                                                   *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Atom =
--- a/src/Tools/Metis/src/Atom.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Atom.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC ATOMS                                                   *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Atom :> Atom =
--- a/src/Tools/Metis/src/AtomNet.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/AtomNet.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC ATOMS              *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature AtomNet =
--- a/src/Tools/Metis/src/AtomNet.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/AtomNet.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC ATOMS              *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure AtomNet :> AtomNet =
--- a/src/Tools/Metis/src/Clause.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Clause.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* CLAUSE = ID + THEOREM                                                     *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Clause =
--- a/src/Tools/Metis/src/Clause.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Clause.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* CLAUSE = ID + THEOREM                                                     *)
-(* Copyright (c) 2002-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Clause :> Clause =
--- a/src/Tools/Metis/src/ElementSet.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/ElementSet.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE SETS WITH A FIXED ELEMENT TYPE                                     *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature ElementSet =
--- a/src/Tools/Metis/src/ElementSet.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/ElementSet.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE SETS WITH A FIXED ELEMENT TYPE                                     *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 functor ElementSet (Key : Ordered) :> ElementSet where type element = Key.t =
--- a/src/Tools/Metis/src/Formula.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Formula.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC FORMULAS                                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Formula =
--- a/src/Tools/Metis/src/Formula.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Formula.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC FORMULAS                                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Formula :> Formula =
--- a/src/Tools/Metis/src/Heap.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Heap.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* A HEAP DATATYPE FOR ML                                                    *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Heap =
--- a/src/Tools/Metis/src/Heap.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Heap.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* A HEAP DATATYPE FOR ML                                                    *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Heap :> Heap =
--- a/src/Tools/Metis/src/KeyMap.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/KeyMap.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE MAPS WITH A FIXED KEY TYPE                                         *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature KeyMap =
--- a/src/Tools/Metis/src/KeyMap.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/KeyMap.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE MAPS WITH A FIXED KEY TYPE                                         *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 functor KeyMap (Key : Ordered) :> KeyMap where type key = Key.t =
--- a/src/Tools/Metis/src/KnuthBendixOrder.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/KnuthBendixOrder.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* THE KNUTH-BENDIX TERM ORDERING                                            *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature KnuthBendixOrder =
--- a/src/Tools/Metis/src/KnuthBendixOrder.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/KnuthBendixOrder.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* KNUTH-BENDIX TERM ORDERING CONSTRAINTS                                    *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure KnuthBendixOrder :> KnuthBendixOrder =
--- a/src/Tools/Metis/src/Lazy.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Lazy.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* SUPPORT FOR LAZY EVALUATION                                               *)
-(* Copyright (c) 2007 Joe Hurd, distributed under the GNU GPL version 2      *)
+(* Copyright (c) 2007 Joe Hurd, distributed under the BSD License      *)
 (* ========================================================================= *)
 
 signature Lazy =
--- a/src/Tools/Metis/src/Lazy.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Lazy.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* SUPPORT FOR LAZY EVALUATION                                               *)
-(* Copyright (c) 2007 Joe Hurd, distributed under the GNU GPL version 2      *)
+(* Copyright (c) 2007 Joe Hurd, distributed under the BSD License      *)
 (* ========================================================================= *)
 
 structure Lazy :> Lazy =
--- a/src/Tools/Metis/src/Literal.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Literal.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC LITERALS                                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Literal =
--- a/src/Tools/Metis/src/Literal.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Literal.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC LITERALS                                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Literal :> Literal =
--- a/src/Tools/Metis/src/LiteralNet.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/LiteralNet.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC LITERALS           *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature LiteralNet =
--- a/src/Tools/Metis/src/LiteralNet.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/LiteralNet.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC LITERALS           *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure LiteralNet :> LiteralNet =
--- a/src/Tools/Metis/src/Map.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Map.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE MAPS                                                               *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Map =
--- a/src/Tools/Metis/src/Map.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Map.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE MAPS                                                               *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Map = RandomMap;
--- a/src/Tools/Metis/src/Model.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Model.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* RANDOM FINITE MODELS                                                      *)
-(* Copyright (c) 2003-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Model =
--- a/src/Tools/Metis/src/Model.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Model.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* RANDOM FINITE MODELS                                                      *)
-(* Copyright (c) 2003-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Model :> Model =
--- a/src/Tools/Metis/src/Name.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Name.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* NAMES                                                                     *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Name =
--- a/src/Tools/Metis/src/Name.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Name.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* NAMES                                                                     *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Name :> Name =
--- a/src/Tools/Metis/src/Normalize.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Normalize.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* NORMALIZING FORMULAS                                                      *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Normalize =
--- a/src/Tools/Metis/src/Normalize.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Normalize.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* NORMALIZING FORMULAS                                                      *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Normalize :> Normalize =
--- a/src/Tools/Metis/src/Options.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Options.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* PROCESSING COMMAND LINE OPTIONS                                           *)
-(* Copyright (c) 2003-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Options =
--- a/src/Tools/Metis/src/Options.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Options.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* PROCESSING COMMAND LINE OPTIONS                                           *)
-(* Copyright (c) 2003-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Options :> Options =
--- a/src/Tools/Metis/src/Ordered.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Ordered.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* ORDERED TYPES                                                             *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Ordered =
--- a/src/Tools/Metis/src/Ordered.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Ordered.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* ORDERED TYPES                                                             *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure IntOrdered =
--- a/src/Tools/Metis/src/Parser.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Parser.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* PARSING AND PRETTY PRINTING                                               *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Parser =
--- a/src/Tools/Metis/src/Parser.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Parser.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* PARSER COMBINATORS                                                        *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Parser :> Parser =
--- a/src/Tools/Metis/src/Portable.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Portable.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* ML SPECIFIC FUNCTIONS                                                     *)
-(* Copyright (c) 2001-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Portable =
--- a/src/Tools/Metis/src/PortableMlton.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/PortableMlton.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* MLTON SPECIFIC FUNCTIONS                                                  *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Portable :> Portable =
--- a/src/Tools/Metis/src/PortableMosml.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/PortableMosml.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* MOSCOW ML SPECIFIC FUNCTIONS                                              *)
-(* Copyright (c) 2002-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Portable :> Portable =
--- a/src/Tools/Metis/src/PortableSmlNJ.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/PortableSmlNJ.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* POLYML SPECIFIC FUNCTIONS                                                 *)
-(* Copyright (c) 2002-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 CM.autoload "$smlnj/init/init.cmi";
--- a/src/Tools/Metis/src/Problem.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Problem.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* SOME SAMPLE PROBLEMS TO TEST PROOF PROCEDURES                             *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Problem =
--- a/src/Tools/Metis/src/Problem.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Problem.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* SOME SAMPLE PROBLEMS TO TEST PROOF PROCEDURES                             *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Problem :> Problem =
--- a/src/Tools/Metis/src/Proof.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Proof.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* PROOFS IN FIRST ORDER LOGIC                                               *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Proof =
--- a/src/Tools/Metis/src/Proof.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Proof.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* PROOFS IN FIRST ORDER LOGIC                                               *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Proof :> Proof =
--- a/src/Tools/Metis/src/RandomMap.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/RandomMap.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE MAPS IMPLEMENTED WITH RANDOMLY BALANCED TREES                      *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure RandomMap :> Map =
--- a/src/Tools/Metis/src/RandomSet.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/RandomSet.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE SETS IMPLEMENTED WITH RANDOMLY BALANCED TREES                      *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure RandomSet :> Set =
--- a/src/Tools/Metis/src/Resolution.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Resolution.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* THE RESOLUTION PROOF PROCEDURE                                            *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Resolution =
--- a/src/Tools/Metis/src/Resolution.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Resolution.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* THE RESOLUTION PROOF PROCEDURE                                            *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Resolution :> Resolution =
--- a/src/Tools/Metis/src/Rewrite.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Rewrite.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* ORDERED REWRITING FOR FIRST ORDER TERMS                                   *)
-(* Copyright (c) 2003-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Rewrite =
--- a/src/Tools/Metis/src/Rewrite.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Rewrite.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* ORDERED REWRITING FOR FIRST ORDER TERMS                                   *)
-(* Copyright (c) 2003-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2003-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Rewrite :> Rewrite =
--- a/src/Tools/Metis/src/Rule.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Rule.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* DERIVED RULES FOR CREATING FIRST ORDER LOGIC THEOREMS                     *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Rule =
--- a/src/Tools/Metis/src/Rule.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Rule.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* DERIVED RULES FOR CREATING FIRST ORDER LOGIC THEOREMS                     *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Rule :> Rule =
--- a/src/Tools/Metis/src/Set.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Set.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE SETS                                                               *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Set =
--- a/src/Tools/Metis/src/Set.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Set.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FINITE SETS                                                               *)
-(* Copyright (c) 2004-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2004-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Set = RandomSet;
--- a/src/Tools/Metis/src/Sharing.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Sharing.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* PRESERVING SHARING OF ML VALUES                                           *)
-(* Copyright (c) 2005-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2005-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Sharing =
--- a/src/Tools/Metis/src/Sharing.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Sharing.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* PRESERVING SHARING OF ML VALUES                                           *)
-(* Copyright (c) 2005-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2005-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Sharing :> Sharing =
--- a/src/Tools/Metis/src/Stream.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Stream.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* A POSSIBLY-INFINITE STREAM DATATYPE FOR ML                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Stream =
--- a/src/Tools/Metis/src/Stream.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Stream.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* A POSSIBLY-INFINITE STREAM DATATYPE FOR ML                                *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Stream :> Stream =
--- a/src/Tools/Metis/src/Subst.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Subst.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC SUBSTITUTIONS                                           *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Subst =
--- a/src/Tools/Metis/src/Subst.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Subst.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC SUBSTITUTIONS                                           *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Subst :> Subst =
--- a/src/Tools/Metis/src/Subsume.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Subsume.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* SUBSUMPTION CHECKING FOR FIRST ORDER LOGIC CLAUSES                        *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Subsume =
--- a/src/Tools/Metis/src/Subsume.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Subsume.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* SUBSUMPTION CHECKING FOR FIRST ORDER LOGIC CLAUSES                        *)
-(* Copyright (c) 2002-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Subsume :> Subsume =
--- a/src/Tools/Metis/src/Term.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Term.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC TERMS                                                   *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Term =
--- a/src/Tools/Metis/src/Term.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Term.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* FIRST ORDER LOGIC TERMS                                                   *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Term :> Term =
--- a/src/Tools/Metis/src/TermNet.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/TermNet.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC TERMS              *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature TermNet =
--- a/src/Tools/Metis/src/TermNet.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/TermNet.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* MATCHING AND UNIFICATION FOR SETS OF FIRST ORDER LOGIC TERMS              *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure TermNet :> TermNet =
--- a/src/Tools/Metis/src/Thm.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Thm.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* A LOGICAL KERNEL FOR FIRST ORDER CLAUSES                                  *)
-(* Copyright (c) 2001-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Thm =
--- a/src/Tools/Metis/src/Thm.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Thm.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* A LOGICAL KERNEL FOR FIRST ORDER CLAUSES                                  *)
-(* Copyright (c) 2001-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Thm :> Thm =
--- a/src/Tools/Metis/src/Tptp.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Tptp.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* INTERFACE TO TPTP PROBLEM FILES                                           *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Tptp =
--- a/src/Tools/Metis/src/Tptp.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Tptp.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* INTERFACE TO TPTP PROBLEM FILES                                           *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Tptp :> Tptp =
--- a/src/Tools/Metis/src/Units.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Units.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* A STORE FOR UNIT THEOREMS                                                 *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Units =
--- a/src/Tools/Metis/src/Units.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Units.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* A STORE FOR UNIT THEOREMS                                                 *)
-(* Copyright (c) 2001-2006 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2006 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Units :> Units =
--- a/src/Tools/Metis/src/Useful.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Useful.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* ML UTILITY FUNCTIONS                                                      *)
-(* Copyright (c) 2001-2005 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2005 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Useful =
--- a/src/Tools/Metis/src/Useful.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Useful.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* ML UTILITY FUNCTIONS                                                      *)
-(* Copyright (c) 2001-2004 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2004 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Useful :> Useful =
--- a/src/Tools/Metis/src/Waiting.sig	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Waiting.sig	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* THE WAITING SET OF CLAUSES                                                *)
-(* Copyright (c) 2002-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 signature Waiting =
--- a/src/Tools/Metis/src/Waiting.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/Waiting.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* THE WAITING SET OF CLAUSES                                                *)
-(* Copyright (c) 2002-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2002-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 structure Waiting :> Waiting =
--- a/src/Tools/Metis/src/problems.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/problems.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* SOME SAMPLE PROBLEMS TO TEST PROOF PROCEDURES                             *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 (* ========================================================================= *)
--- a/src/Tools/Metis/src/problems2tptp.sml	Wed Jun 27 11:06:43 2007 +0200
+++ b/src/Tools/Metis/src/problems2tptp.sml	Wed Jun 27 12:41:36 2007 +0200
@@ -1,6 +1,6 @@
 (* ========================================================================= *)
 (* SOME SAMPLE PROBLEMS TO TEST PROOF PROCEDURES                             *)
-(* Copyright (c) 2001-2007 Joe Hurd, distributed under the GNU GPL version 2 *)
+(* Copyright (c) 2001-2007 Joe Hurd, distributed under the BSD License *)
 (* ========================================================================= *)
 
 open Useful;