doc-src/IsarImplementation/Thy/Prelim.thy
changeset 39876 1ff9bce085bd
parent 39866 5ec01d5acd0c
child 40126 916cb4a28ffd
equal deleted inserted replaced
39875:648c930125f6 39876:1ff9bce085bd
   563   end-users using existing notation for attributes (cf.\
   563   end-users using existing notation for attributes (cf.\
   564   \secref{sec:attributes}).
   564   \secref{sec:attributes}).
   565 
   565 
   566   For example, the predefined configuration option @{attribute
   566   For example, the predefined configuration option @{attribute
   567   show_types} controls output of explicit type constraints for
   567   show_types} controls output of explicit type constraints for
   568   variables in printed terms (cf.\ \secref{sec:parse-print}).  Its
   568   variables in printed terms (cf.\ \secref{sec:read-print}).  Its
   569   value can be modified within Isar text like this:
   569   value can be modified within Isar text like this:
   570 *}
   570 *}
   571 
   571 
   572 declare [[show_types = false]]
   572 declare [[show_types = false]]
   573   -- {* declaration within (local) theory context *}
   573   -- {* declaration within (local) theory context *}