doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 41505 6d19301074cf
parent 41396 5379e4a85a66
child 41506 4c717333b0cc
--- a/doc-src/IsarRef/Thy/HOL_Specific.thy	Mon Jan 10 22:03:24 2011 +0100
+++ b/doc-src/IsarRef/Thy/HOL_Specific.thy	Tue Jan 11 14:12:37 2011 +0100
@@ -388,17 +388,17 @@
 
 text {*
   \begin{matharray}{rcl}
-    @{command_def (HOL) "type_lifting"} & : & @{text "local_theory \<rightarrow> proof(prove)"}
+    @{command_def (HOL) "enriched_type"} & : & @{text "local_theory \<rightarrow> proof(prove)"}
   \end{matharray}
 
   \begin{rail}
-    'type_lifting' (prefix ':')? term
+    'enriched_type' (prefix ':')? term
     ;
   \end{rail}
 
   \begin{description}
 
-  \item @{command (HOL) "type_lifting"} allows to prove and register
+  \item @{command (HOL) "enriched_type"} allows to prove and register
   properties about type constructors which refer to their functorial
   structure; these properties then can be used by other packages to
   deal with those type constructors in certain type constructions.