src/HOL/MicroJava/Comp/TranslCompTp.thy
changeset 60773 d09c66a0ea10
parent 60304 3f429b7d8eb5
child 80914 d97fdabd9e2b
--- a/src/HOL/MicroJava/Comp/TranslCompTp.thy	Thu Jul 23 16:40:47 2015 +0200
+++ b/src/HOL/MicroJava/Comp/TranslCompTp.thy	Thu Jul 23 22:13:42 2015 +0200
@@ -8,7 +8,9 @@
 
 (**********************************************************************)
 
-definition comb :: "['a \<Rightarrow> 'b list \<times> 'c, 'c \<Rightarrow> 'b list \<times> 'd, 'a] \<Rightarrow> 'b list \<times> 'd" where 
+definition comb :: "['a \<Rightarrow> 'b list \<times> 'c, 'c \<Rightarrow> 'b list \<times> 'd, 'a] \<Rightarrow> 'b list \<times> 'd"
+  (infixr "\<box>" 55)
+where 
   "comb == (\<lambda> f1 f2 x0. let (xs1, x1) = f1 x0; 
                             (xs2, x2) = f2 x1 
                         in  (xs1 @ xs2, x2))"
@@ -16,9 +18,6 @@
 definition comb_nil :: "'a \<Rightarrow> 'b list \<times> 'a" where
   "comb_nil a == ([], a)"
 
-notation (xsymbols)
-  comb  (infixr "\<box>" 55)
-
 lemma comb_nil_left [simp]: "comb_nil \<box> f = f"
   by (simp add: comb_def comb_nil_def split_beta)