changeset 22838 | 466599ecf610 |
parent 22744 | 5cbe966d67a2 |
child 22921 | 475ff421a6a3 |
--- a/src/HOL/Library/ExecutableSet.thy Sun May 06 18:07:06 2007 +0200 +++ b/src/HOL/Library/ExecutableSet.thy Sun May 06 21:49:23 2007 +0200 @@ -347,7 +347,7 @@ "insert" ("{*insertl*}") "op Un" ("{*unionl*}") "op Int" ("{*intersect*}") - "HOL.minus" :: "'a set \<Rightarrow> 'a set \<Rightarrow> 'a set" + "minus" :: "'a set \<Rightarrow> 'a set \<Rightarrow> 'a set" ("{*flip subtract*}") "image" ("{*map_distinct*}") "Union" ("{*unions*}")