corrected slip
authorhaftmann
Sat, 07 Jan 2012 11:45:53 +0100
changeset 46151 913ea585efdc
parent 46150 d6cafcc012ec
child 46152 793cecd4ffc0
corrected slip
src/HOL/List.thy
--- a/src/HOL/List.thy	Sat Jan 07 09:32:18 2012 +0100
+++ b/src/HOL/List.thy	Sat Jan 07 11:45:53 2012 +0100
@@ -5216,10 +5216,10 @@
   by (simp add: member_def)
 
 definition list_all :: "('a \<Rightarrow> bool) \<Rightarrow> 'a list \<Rightarrow> bool" where
-  [code_abbrev]: list_all_iff: "list_all P xs \<longleftrightarrow> Ball (set xs) P"
+  list_all_iff [code_abbrev]: "list_all P xs \<longleftrightarrow> Ball (set xs) P"
 
 definition list_ex :: "('a \<Rightarrow> bool) \<Rightarrow> 'a list \<Rightarrow> bool" where
-  [code_abbrev]: list_ex_iff: "list_ex P xs \<longleftrightarrow> Bex (set xs) P"
+  list_ex_iff [code_abbrev]: "list_ex P xs \<longleftrightarrow> Bex (set xs) P"
 
 definition list_ex1 :: "('a \<Rightarrow> bool) \<Rightarrow> 'a list \<Rightarrow> bool" where
   list_ex1_iff [code_abbrev]: "list_ex1 P xs \<longleftrightarrow> (\<exists>! x. x \<in> set xs \<and> P x)"