src/HOL/NanoJava/Equivalence.thy
changeset 14565 c6dc17aab88a
parent 14174 f3cafd2929d5
child 16417 9bc16273c2d4
--- a/src/HOL/NanoJava/Equivalence.thy	Wed Apr 14 13:28:46 2004 +0200
+++ b/src/HOL/NanoJava/Equivalence.thy	Wed Apr 14 14:13:05 2004 +0200
@@ -166,6 +166,8 @@
          "MGTe e Z \<equiv> (\<lambda>s. Z = s, e, \<lambda>v t. \<exists>n. Z -e>v-n-> t)"
 syntax (xsymbols)
          MGTe    :: "expr => state => etriple" ("MGT\<^sub>e")
+syntax (HTML output)
+         MGTe    :: "expr => state => etriple" ("MGT\<^sub>e")
 
 lemma MGF_implies_complete:
  "\<forall>Z. {} |\<turnstile> { MGT c Z} \<Longrightarrow> \<Turnstile>  {P} c {Q} \<Longrightarrow> {} \<turnstile>  {P} c {Q}"