doc-src/IsarImplementation/Thy/prelim.thy
changeset 24137 8d7896398147
parent 22869 9f915d44a666
child 26864 1417e704d724
--- a/doc-src/IsarImplementation/Thy/prelim.thy	Thu Aug 02 23:18:13 2007 +0200
+++ b/doc-src/IsarImplementation/Thy/prelim.thy	Fri Aug 03 16:28:15 2007 +0200
@@ -156,8 +156,8 @@
   \end{mldecls}
   \begin{mldecls}
   @{index_ML_type theory_ref} \\
-  @{index_ML Theory.self_ref: "theory -> theory_ref"} \\
   @{index_ML Theory.deref: "theory_ref -> theory"} \\
+  @{index_ML Theory.check_thy: "theory -> theory_ref"} \\
   \end{mldecls}
 
   \begin{description}
@@ -187,12 +187,14 @@
   always valid theory; updates on the original are propagated
   automatically.
 
-  \item @{ML "Theory.self_ref"}~@{text "thy"} and @{ML
-  "Theory.deref"}~@{text "thy_ref"} convert between @{ML_type
-  "theory"} and @{ML_type "theory_ref"}.  As the referenced theory
-  evolves monotonically over time, later invocations of @{ML
+  \item @{ML "Theory.deref"}~@{text "thy_ref"} turns a @{ML_type
+  "theory_ref"} into an @{ML_type "theory"} value.  As the referenced
+  theory evolves monotonically over time, later invocations of @{ML
   "Theory.deref"} may refer to a larger context.
 
+  \item @{ML "Theory.check_thy"}~@{text "thy"} produces a @{ML_type
+  "theory_ref"} from a valid @{ML_type "theory"} value.
+
   \end{description}
 *}