src/Doc/Isar_Ref/Spec.thy
changeset 59422 db6ecef63d5b
parent 59320 a375de4dc07a
child 59781 a71dbf3481a2
equal deleted inserted replaced
59421:cefeea956989 59422:db6ecef63d5b
   913     @@{command instance} (() | (@{syntax nameref} + @'and') '::' @{syntax arity} |
   913     @@{command instance} (() | (@{syntax nameref} + @'and') '::' @{syntax arity} |
   914       @{syntax nameref} ('<' | '\<subseteq>') @{syntax nameref} )
   914       @{syntax nameref} ('<' | '\<subseteq>') @{syntax nameref} )
   915     ;
   915     ;
   916     @@{command subclass} @{syntax target}? @{syntax nameref}
   916     @@{command subclass} @{syntax target}? @{syntax nameref}
   917     ;
   917     ;
   918     @@{command class_deps} @{syntax sort}? @{syntax sort}?
   918     @@{command class_deps} ( ( @{syntax sort} | ( '(' ( @{syntax sort} + @'|' ) ')' ) ) \<newline>
       
   919       ( @{syntax sort} | ( '(' ( @{syntax sort} + @'|' ) ')' ) )? )?
   919   \<close>}
   920   \<close>}
   920 
   921 
   921   \begin{description}
   922   \begin{description}
   922 
   923 
   923   \item @{command "class"}~@{text "c = superclasses + body"} defines
   924   \item @{command "class"}~@{text "c = superclasses + body"} defines
   977 
   978 
   978   \item @{command "print_classes"} prints all classes in the current
   979   \item @{command "print_classes"} prints all classes in the current
   979   theory.
   980   theory.
   980 
   981 
   981   \item @{command "class_deps"} visualizes all classes and their
   982   \item @{command "class_deps"} visualizes all classes and their
   982   subclass relations as a Hasse diagram.  An optional first sort argument
   983   subclass relations as a Hasse diagram.  An optional first argument
   983   constrains the set of classes to all subclasses of this sort,
   984   constrains the set of classes to all subclasses of at least one given
   984   an optional second sort argument to all superclasses of this sort.
   985   sort, an optional second rgument to all superclasses of at least one given
       
   986   sort.
   985 
   987 
   986   \item @{method intro_classes} repeatedly expands all class
   988   \item @{method intro_classes} repeatedly expands all class
   987   introduction rules of this theory.  Note that this method usually
   989   introduction rules of this theory.  Note that this method usually
   988   needs not be named explicitly, as it is already included in the
   990   needs not be named explicitly, as it is already included in the
   989   default proof step (e.g.\ of @{command "proof"}).  In particular,
   991   default proof step (e.g.\ of @{command "proof"}).  In particular,