src/HOL/Set.thy
changeset 20380 14f9f2a1caa6
parent 20217 25b068a99d2b
child 21210 c17fd2df4e9e
--- a/src/HOL/Set.thy	Mon Aug 14 13:46:05 2006 +0200
+++ b/src/HOL/Set.thy	Mon Aug 14 13:46:06 2006 +0200
@@ -2258,10 +2258,4 @@
   ord_eq_less_trans
   trans
 
-subsection {* Code generator setup *}
-
-code_alias
-  "op Int" "Set.inter"
-  "op Un" "Set.union"
-
 end