src/HOL/Library/List_Prefix.thy
changeset 21404 eb85850d3eb7
parent 21305 d41eddfd2b66
child 22178 29b95968272b
--- a/src/HOL/Library/List_Prefix.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/Library/List_Prefix.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -159,7 +159,7 @@
 subsection {* Parallel lists *}
 
 definition
-  parallel :: "'a list => 'a list => bool"    (infixl "\<parallel>" 50)
+  parallel :: "'a list => 'a list => bool"  (infixl "\<parallel>" 50) where
   "(xs \<parallel> ys) = (\<not> xs \<le> ys \<and> \<not> ys \<le> xs)"
 
 lemma parallelI [intro]: "\<not> xs \<le> ys ==> \<not> ys \<le> xs ==> xs \<parallel> ys"
@@ -218,7 +218,7 @@
 subsection {* Postfix order on lists *}
 
 definition
-  postfix :: "'a list => 'a list => bool"  ("(_/ >>= _)" [51, 50] 50)
+  postfix :: "'a list => 'a list => bool"  ("(_/ >>= _)" [51, 50] 50) where
   "(xs >>= ys) = (\<exists>zs. xs = zs @ ys)"
 
 lemma postfixI [intro?]: "xs = zs @ ys ==> xs >>= ys"