diff -r 66893c47500d -r 701912f5645a src/CCL/Set.thy --- a/src/CCL/Set.thy Fri Aug 23 22:47:51 2024 +0200 +++ b/src/CCL/Set.thy Fri Aug 23 23:14:39 2024 +0200 @@ -21,6 +21,8 @@ "_Coll" :: "[idt, o] \ 'a set" ("(1{_./ _})") translations "{x. P}" == "CONST Collect(\x. P)" +syntax_consts + "_Coll" == Collect lemma CollectI: "P(a) \ a : {x. P(x)}" apply (rule mem_Collect_iff [THEN iffD2]) @@ -53,6 +55,9 @@ translations "ALL x:A. P" == "CONST Ball(A, \x. P)" "EX x:A. P" == "CONST Bex(A, \x. P)" +syntax_consts + "_Ball" == Ball and + "_Bex" == Bex lemma ballI: "(\x. x:A \ P(x)) \ ALL x:A. P(x)" by (simp add: Ball_def) @@ -127,6 +132,9 @@ translations "INT x:A. B" == "CONST INTER(A, \x. B)" "UN x:A. B" == "CONST UNION(A, \x. B)" +syntax_consts + "_INTER" == INTER and + "_UNION" == UNION definition Inter :: "(('a set)set) \ 'a set" where "Inter(S) == (INT x:S. x)"