src/HOL/BNF/Examples/Derivation_Trees/Parallel.thy
changeset 54538 ba7392b52a7c
parent 49882 946efb120c42
--- a/src/HOL/BNF/Examples/Derivation_Trees/Parallel.thy	Wed Nov 20 18:32:25 2013 +0100
+++ b/src/HOL/BNF/Examples/Derivation_Trees/Parallel.thy	Wed Nov 20 18:58:00 2013 +0100
@@ -12,7 +12,6 @@
 begin
 
 no_notation plus_class.plus (infixl "+" 65)
-no_notation Sublist.parallel (infixl "\<parallel>" 50)
 
 consts Nplus :: "N \<Rightarrow> N \<Rightarrow> N" (infixl "+" 60)
 
@@ -145,4 +144,4 @@
   thus ?thesis by blast
 qed
 
-end
\ No newline at end of file
+end