TFL/thry.sml
changeset 9867 bf8300fa4238
parent 8416 8eb32cd3122e
--- a/TFL/thry.sml	Tue Sep 05 18:53:21 2000 +0200
+++ b/TFL/thry.sml	Tue Sep 05 18:53:42 2000 +0200
@@ -1,9 +1,30 @@
-(*  Title:      TFL/thry
+(*  Title:      TFL/thry.sml
     ID:         $Id$
     Author:     Konrad Slind, Cambridge University Computer Laboratory
     Copyright   1997  University of Cambridge
 *)
 
+signature Thry_sig =
+sig
+  val match_term : theory -> term -> term 
+                    -> (term*term)list * (typ*typ)list
+
+  val match_type : theory -> typ -> typ -> (typ*typ)list
+
+  val typecheck : theory -> term -> cterm
+
+  (* Datatype facts of various flavours *)
+  val match_info: theory -> string -> {constructors:term list,
+                                     case_const:term} option
+
+  val induct_info: theory -> string -> {constructors:term list,
+                                      nchotomy:thm} option
+
+  val extract_info: theory -> {case_congs:thm list, case_rewrites:thm list}
+
+end;
+
+
 structure Thry : Thry_sig (* LThry_sig *) = 
 struct