src/Doc/IsarRef/Spec.thy
changeset 51565 5e9fdbdf88ce
parent 51313 102a0a0718c5
child 51585 fcd5af4aac2b
equal deleted inserted replaced
51564:bfdc3f720bd6 51565:5e9fdbdf88ce
   699 
   699 
   700   \item @{command "print_dependencies"}~@{text "expr"} is useful for
   700   \item @{command "print_dependencies"}~@{text "expr"} is useful for
   701   understanding the effect of an interpretation of @{text "expr"}.  It
   701   understanding the effect of an interpretation of @{text "expr"}.  It
   702   lists all locale instances for which interpretations would be added
   702   lists all locale instances for which interpretations would be added
   703   to the current context.  Variant @{command
   703   to the current context.  Variant @{command
   704   "print_dependencies"}@{text "!"} prints all locale instances that
   704   "print_dependencies"}@{text "!"} does not generalize parameters and
   705   would be considered for interpretation, and would be interpreted in
   705   assumes an empty context --- that is, it prints all locale instances
   706   an empty context (that is, without interpretations).
   706   that would be considered for interpretation.  The latter is useful
       
   707   for understanding the dependencies of a locale expression.
   707 
   708 
   708   \item @{command "print_interps"}~@{text "locale"} lists all
   709   \item @{command "print_interps"}~@{text "locale"} lists all
   709   interpretations of @{text "locale"} in the current theory or proof
   710   interpretations of @{text "locale"} in the current theory or proof
   710   context, including those due to a combination of a @{command
   711   context, including those due to a combination of an @{command
   711   "interpretation"} or @{command "interpret"} and one or several
   712   "interpretation"} or @{command "interpret"} and one or several
   712   @{command "sublocale"} declarations.
   713   @{command "sublocale"} declarations.
   713 
   714 
   714   \end{description}
   715   \end{description}
   715 
   716