src/HOL/IMP/Natural.thy
changeset 14565 c6dc17aab88a
parent 12546 0c90e581379f
child 16417 9bc16273c2d4
--- a/src/HOL/IMP/Natural.thy	Wed Apr 14 13:28:46 2004 +0200
+++ b/src/HOL/IMP/Natural.thy	Wed Apr 14 14:13:05 2004 +0200
@@ -17,6 +17,9 @@
 syntax (xsymbols)
   "_evalc" :: "[com,state,state] \<Rightarrow> bool" ("\<langle>_,_\<rangle>/ \<longrightarrow>\<^sub>c _" [0,0,60] 60)
 
+syntax (HTML output)
+  "_evalc" :: "[com,state,state] \<Rightarrow> bool" ("\<langle>_,_\<rangle>/ \<longrightarrow>\<^sub>c _" [0,0,60] 60)
+
 text {*
   We write @{text "\<langle>c,s\<rangle> \<longrightarrow>\<^sub>c s'"} for \emph{Statement @{text c}, started 
   in state @{text s}, terminates in state @{text s'}}. Formally,