src/Doc/IsarRef/Spec.thy
changeset 50716 e04c44dc11fc
parent 50128 599c935aac82
child 51313 102a0a0718c5
equal deleted inserted replaced
50715:8cfd585b9162 50716:e04c44dc11fc
   457 text {*
   457 text {*
   458   \begin{matharray}{rcl}
   458   \begin{matharray}{rcl}
   459     @{command_def "locale"} & : & @{text "theory \<rightarrow> local_theory"} \\
   459     @{command_def "locale"} & : & @{text "theory \<rightarrow> local_theory"} \\
   460     @{command_def "print_locale"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
   460     @{command_def "print_locale"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
   461     @{command_def "print_locales"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
   461     @{command_def "print_locales"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
       
   462     @{command_def "locale_deps"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
   462     @{method_def intro_locales} & : & @{text method} \\
   463     @{method_def intro_locales} & : & @{text method} \\
   463     @{method_def unfold_locales} & : & @{text method} \\
   464     @{method_def unfold_locales} & : & @{text method} \\
   464   \end{matharray}
   465   \end{matharray}
   465 
   466 
   466   \indexisarelem{fixes}\indexisarelem{constrains}\indexisarelem{assumes}
   467   \indexisarelem{fixes}\indexisarelem{constrains}\indexisarelem{assumes}
   569   elements by default.  Use @{command "print_locale"}@{text "!"} to
   570   elements by default.  Use @{command "print_locale"}@{text "!"} to
   570   have them included.
   571   have them included.
   571 
   572 
   572   \item @{command "print_locales"} prints the names of all locales
   573   \item @{command "print_locales"} prints the names of all locales
   573   of the current theory.
   574   of the current theory.
       
   575 
       
   576   \item @{command "locale_deps"} visualizes all locales and their
       
   577   relations as a Hasse diagram. This includes locales defined as type
       
   578   classes (\secref{sec:class}).
   574 
   579 
   575   \item @{method intro_locales} and @{method unfold_locales}
   580   \item @{method intro_locales} and @{method unfold_locales}
   576   repeatedly expand all introduction rules of locale predicates of the
   581   repeatedly expand all introduction rules of locale predicates of the
   577   theory.  While @{method intro_locales} only applies the @{text
   582   theory.  While @{method intro_locales} only applies the @{text
   578   loc.intro} introduction rules and therefore does not decend to
   583   loc.intro} introduction rules and therefore does not decend to