src/HOL/Induct/SList.thy
changeset 23029 79ee75dc1e59
parent 22267 ea31e6ea0e2e
child 23235 eb365b39b36d
--- a/src/HOL/Induct/SList.thy	Sat May 19 11:33:34 2007 +0200
+++ b/src/HOL/Induct/SList.thy	Sat May 19 11:33:57 2007 +0200
@@ -159,6 +159,10 @@
   map       :: "('a=>'b) => ('a list => 'b list)" where
   "map f xs = list_rec xs [] (%x l r. f(x)#r)"
 
+no_syntax
+  append :: "'a list => 'a list => 'a list" (infixr "@" 65)
+hide const "List.append"
+
 definition
   append    :: "['a list, 'a list] => 'a list"   (infixr "@" 65) where
   "xs@ys = list_rec xs ys (%x l r. x#r)"