src/Doc/Isar_Ref/Spec.thy
changeset 58202 be1d10595b7b
parent 57947 189d421ca72d
child 58305 57752a91eec4
equal deleted inserted replaced
58201:5bf56c758e02 58202:be1d10595b7b
   830     ;
   830     ;
   831     @@{command instance} (() | (@{syntax nameref} + @'and') '::' @{syntax arity} |
   831     @@{command instance} (() | (@{syntax nameref} + @'and') '::' @{syntax arity} |
   832       @{syntax nameref} ('<' | '\<subseteq>') @{syntax nameref} )
   832       @{syntax nameref} ('<' | '\<subseteq>') @{syntax nameref} )
   833     ;
   833     ;
   834     @@{command subclass} @{syntax target}? @{syntax nameref}
   834     @@{command subclass} @{syntax target}? @{syntax nameref}
       
   835     ;
       
   836     @@{command class_deps} @{syntax sort}? @{syntax sort}?
   835   \<close>}
   837   \<close>}
   836 
   838 
   837   \begin{description}
   839   \begin{description}
   838 
   840 
   839   \item @{command "class"}~@{text "c = superclasses + body"} defines
   841   \item @{command "class"}~@{text "c = superclasses + body"} defines
   893 
   895 
   894   \item @{command "print_classes"} prints all classes in the current
   896   \item @{command "print_classes"} prints all classes in the current
   895   theory.
   897   theory.
   896 
   898 
   897   \item @{command "class_deps"} visualizes all classes and their
   899   \item @{command "class_deps"} visualizes all classes and their
   898   subclass relations as a Hasse diagram.
   900   subclass relations as a Hasse diagram.  An optional first sort argument
       
   901   constrains the set of classes to all subclasses of this sort,
       
   902   an optional second sort argument to all superclasses of this sort.
   899 
   903 
   900   \item @{method intro_classes} repeatedly expands all class
   904   \item @{method intro_classes} repeatedly expands all class
   901   introduction rules of this theory.  Note that this method usually
   905   introduction rules of this theory.  Note that this method usually
   902   needs not be named explicitly, as it is already included in the
   906   needs not be named explicitly, as it is already included in the
   903   default proof step (e.g.\ of @{command "proof"}).  In particular,
   907   default proof step (e.g.\ of @{command "proof"}).  In particular,