doc-src/IsarImplementation/Thy/Logic.thy
changeset 47174 b9b2e183e94d
parent 46497 89ccf66aa73d
child 47498 e3fc50c7da13
--- a/doc-src/IsarImplementation/Thy/Logic.thy	Wed Mar 28 11:04:39 2012 +0200
+++ b/doc-src/IsarImplementation/Thy/Logic.thy	Wed Mar 28 11:17:32 2012 +0200
@@ -127,8 +127,7 @@
   \begin{mldecls}
   @{index_ML Sign.subsort: "theory -> sort * sort -> bool"} \\
   @{index_ML Sign.of_sort: "theory -> typ * sort -> bool"} \\
-  @{index_ML Sign.add_types: "Proof.context ->
-  (binding * int * mixfix) list -> theory -> theory"} \\
+  @{index_ML Sign.add_type: "Proof.context -> binding * int * mixfix -> theory -> theory"} \\
   @{index_ML Sign.add_type_abbrev: "Proof.context ->
   binding * string list * typ -> theory -> theory"} \\
   @{index_ML Sign.primitive_class: "binding * class list -> theory -> theory"} \\
@@ -166,7 +165,7 @@
   \item @{ML Sign.of_sort}~@{text "thy (\<tau>, s)"} tests whether type
   @{text "\<tau>"} is of sort @{text "s"}.
 
-  \item @{ML Sign.add_types}~@{text "ctxt [(\<kappa>, k, mx), \<dots>]"} declares a
+  \item @{ML Sign.add_type}~@{text "ctxt (\<kappa>, k, mx)"} declares a
   new type constructors @{text "\<kappa>"} with @{text "k"} arguments and
   optional mixfix syntax.