src/Doc/Isar_Ref/Spec.thy
changeset 58202 be1d10595b7b
parent 57947 189d421ca72d
child 58305 57752a91eec4
--- a/src/Doc/Isar_Ref/Spec.thy	Sun Sep 07 17:51:28 2014 +0200
+++ b/src/Doc/Isar_Ref/Spec.thy	Sun Sep 07 17:51:32 2014 +0200
@@ -832,6 +832,8 @@
       @{syntax nameref} ('<' | '\<subseteq>') @{syntax nameref} )
     ;
     @@{command subclass} @{syntax target}? @{syntax nameref}
+    ;
+    @@{command class_deps} @{syntax sort}? @{syntax sort}?
   \<close>}
 
   \begin{description}
@@ -895,7 +897,9 @@
   theory.
 
   \item @{command "class_deps"} visualizes all classes and their
-  subclass relations as a Hasse diagram.
+  subclass relations as a Hasse diagram.  An optional first sort argument
+  constrains the set of classes to all subclasses of this sort,
+  an optional second sort argument to all superclasses of this sort.
 
   \item @{method intro_classes} repeatedly expands all class
   introduction rules of this theory.  Note that this method usually