src/Doc/System/Sessions.thy
changeset 69610 10644973cdde
parent 69603 67ae2e164c0f
child 69671 2486792eaf61
equal deleted inserted replaced
69609:1d2d4ae9ab81 69610:10644973cdde
   719   \<^medskip> The following update options are supported:
   719   \<^medskip> The following update options are supported:
   720 
   720 
   721     \<^item> @{system_option update_inner_syntax_cartouches} to update inner syntax
   721     \<^item> @{system_option update_inner_syntax_cartouches} to update inner syntax
   722     (types, terms, etc.)~to use cartouches, instead of double-quoted strings
   722     (types, terms, etc.)~to use cartouches, instead of double-quoted strings
   723     or atomic identifiers. For example, ``\<^theory_text>\<open>lemma \<doublequote>x =
   723     or atomic identifiers. For example, ``\<^theory_text>\<open>lemma \<doublequote>x =
   724     x\<doublequote>\<close>'' is replaced by ``\<^theory_text>\<open>lemma \<open>x = x\<close>\<close>'', and ``\<^theory_text>\<open>fix x\<close>''
   724     x\<doublequote>\<close>'' is replaced by ``\<^theory_text>\<open>lemma \<open>x = x\<close>\<close>'', and ``\<^theory_text>\<open>assume
   725     is replaced by ``\<^theory_text>\<open>fix \<open>x\<close>\<close>''.
   725     A\<close>'' is replaced by ``\<^theory_text>\<open>assume \<open>A\<close>\<close>''.
   726 
   726 
   727     \<^item> @{system_option update_mixfix_cartouches} to update mixfix templates to
   727     \<^item> @{system_option update_mixfix_cartouches} to update mixfix templates to
   728     use cartouches instead of double-quoted strings. For example, ``\<^theory_text>\<open>(infixl
   728     use cartouches instead of double-quoted strings. For example, ``\<^theory_text>\<open>(infixl
   729     \<doublequote>+\<doublequote> 65)\<close>'' is replaced by ``\<^theory_text>\<open>(infixl \<open>+\<close>
   729     \<doublequote>+\<doublequote> 65)\<close>'' is replaced by ``\<^theory_text>\<open>(infixl \<open>+\<close>
   730     65)\<close>''.
   730     65)\<close>''.