doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 45767 fe2fd2f76f48
parent 45701 615da8b8d758
child 45768 97be233b32ed
--- a/doc-src/IsarRef/Thy/HOL_Specific.thy	Mon Dec 05 07:31:11 2011 +0100
+++ b/doc-src/IsarRef/Thy/HOL_Specific.thy	Mon Dec 05 14:44:46 2011 +0100
@@ -1264,10 +1264,6 @@
      (@'morphisms' @{syntax name} @{syntax name})?; 
   "}
 
- The injection from a quotient type to a raw type is called @{text rep_t},
-  its inverse @{text abs_t} unless explicit @{keyword (HOL)
-  "morphisms"} specification provides alternative names.
-
   @{rail "
     @@{command (HOL) quotient_definition} constdecl? @{syntax thmdecl}? \\
     @{syntax term} 'is' @{syntax term};
@@ -1277,7 +1273,9 @@
 
   \begin{description}
   
-  \item @{command (HOL) "quotient_type"} defines quotient types.
+  \item @{command (HOL) "quotient_type"} defines quotient types. The injection from a quotient type 
+  to a raw type is called @{text rep_t}, its inverse @{text abs_t} unless explicit @{keyword (HOL)
+  "morphisms"} specification provides alternative names.
 
   \item @{command (HOL) "quotient_definition"} defines a constant on the quotient type.