changeset 2412 | 025e80ed698d |
parent 2393 | 651fce76c86c |
child 2684 | 9781d63ef063 |
--- a/src/HOL/Set.thy Mon Dec 16 10:29:30 1996 +0100 +++ b/src/HOL/Set.thy Mon Dec 16 10:35:01 1996 +0100 @@ -110,6 +110,9 @@ "*Ball" :: [pttrn, 'a set, bool] => bool ("(3\\<forall> _\\<in>_./ _)" [0, 0, 10] 10) "*Bex" :: [pttrn, 'a set, bool] => bool ("(3\\<exists> _\\<in>_./ _)" [0, 0, 10] 10) +translations + "op \\<subseteq>" => "op <=" + (** Rules and definitions **)