doc-src/IsarRef/Thy/Misc.thy
changeset 28779 698960f08652
parent 28778 a25630deacaf
child 29893 defab1c6a6b5
--- a/doc-src/IsarRef/Thy/Misc.thy	Thu Nov 13 22:01:30 2008 +0100
+++ b/doc-src/IsarRef/Thy/Misc.thy	Thu Nov 13 22:02:18 2008 +0100
@@ -4,7 +4,7 @@
 imports Main
 begin
 
-chapter {* Other commands \label{ch:pure-syntax} *}
+chapter {* Other commands *}
 
 section {* Inspecting the context *}
 
@@ -12,7 +12,6 @@
   \begin{matharray}{rcl}
     @{command_def "print_commands"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
     @{command_def "print_theory"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
-    @{command_def "print_syntax"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
     @{command_def "print_methods"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
     @{command_def "print_attributes"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
     @{command_def "print_theorems"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
@@ -48,11 +47,6 @@
   the theory context; the ``@{text "!"}'' option indicates extra
   verbosity.
 
-  \item @{command "print_syntax"} prints the inner syntax of types and
-  terms, depending on the current context.  The output can be very
-  verbose, including grammar tables and syntax translation rules.  See
-  \chref{ch:inner-syntax} for further information on inner syntax.
-  
   \item @{command "print_methods"} prints all proof methods
   available in the current theory context.