doc-src/Ref/classical.tex
changeset 4561 19f1a01570bf
parent 4507 f313d8fb8f49
child 4597 a0bdee64194c
--- a/doc-src/Ref/classical.tex	Mon Jan 12 17:48:55 1998 +0100
+++ b/doc-src/Ref/classical.tex	Mon Jan 12 17:49:12 1998 +0100
@@ -558,12 +558,22 @@
 \end{ttdescription}
 
 \subsection{The current claset}\label{sec:current-claset}
-Some logics (\FOL, {\HOL} and \ZF) support the concept of a current
-claset\index{claset!current}.  This is a default set of classical rules.  The
-underlying idea is quite similar to that of a current simpset described in
-\S\ref{sec:simp-for-dummies}; please read that section, including its
-warnings.  Just like simpsets, clasets can be associated with theories.  The
-tactics
+
+Each theory is equipped with an implicit \emph{current
+  claset}\index{claset!current}.  This is a default set of classical
+rules.  The underlying idea is quite similar to that of a current
+simpset described in \S\ref{sec:simp-for-dummies}; please read that
+section, including its warnings.  The implicit claset can be accessed
+as follows:
+\begin{ttbox}
+claset        : unit -> claset
+claset_ref    : unit -> claset ref
+claset_of     : theory -> claset
+claset_ref_of : theory -> claset ref
+print_claset  : theory -> unit
+\end{ttbox}
+
+The tactics
 \begin{ttbox}
 Blast_tac        : int -> tactic
 Auto_tac         :        tactic
@@ -584,10 +594,10 @@
 \indexbold{*Step_tac}
 make use of the current claset.  For example, \texttt{Blast_tac} is defined as 
 \begin{ttbox}
-fun Blast_tac i st = blast_tac (!claset) i st;
+fun Blast_tac i st = blast_tac (claset()) i st;
 \end{ttbox}
-and gets the current claset, \ttindex{!claset}, only after it is applied to a
-proof state.  The functions
+and gets the current claset, only after it is applied to a proof
+state.  The functions
 \begin{ttbox}
 AddSIs, AddSEs, AddSDs, AddIs, AddEs, AddDs: thm list -> unit
 \end{ttbox}