doc-src/TutorialI/Documents/Documents.thy
changeset 25399 595da5b9854b
parent 25338 6eb185959aec
child 26698 ca558202ffa5
equal deleted inserted replaced
25398:35f600d9bf06 25399:595da5b9854b
   174 (*<*)
   174 (*<*)
   175 local
   175 local
   176 (*>*)
   176 (*>*)
   177 
   177 
   178 text {*The \commdx{notation} command associates a mixfix
   178 text {*The \commdx{notation} command associates a mixfix
   179 annotation with a logical constant.  The print mode specification of
   179 annotation with a known constant.  The print mode specification of
   180 \isakeyword{syntax}, here @{text "(xsymbols)"}, is optional.
   180 \isakeyword{syntax}, here @{text "(xsymbols)"}, is optional.
   181 
   181 
   182 We may now write @{text "A [+] B"} or @{text "A \<oplus> B"} in input, while
   182 We may now write @{text "A [+] B"} or @{text "A \<oplus> B"} in input, while
   183 output uses the nicer syntax of $xsymbols$ whenever that print mode is
   183 output uses the nicer syntax of $xsymbols$ whenever that print mode is
   184 active.  Such an arrangement is particularly useful for interactive
   184 active.  Such an arrangement is particularly useful for interactive