diff -r fad60fe1565c -r 98d380757893 src/HOL/Set.thy --- a/src/HOL/Set.thy Fri Jan 13 01:13:17 2006 +0100 +++ b/src/HOL/Set.thy Fri Jan 13 14:43:09 2006 +0100 @@ -64,6 +64,8 @@ "_Ball" :: "pttrn => 'a set => bool => bool" ("(3ALL _:_./ _)" [0, 0, 10] 10) "_Bex" :: "pttrn => 'a set => bool => bool" ("(3EX _:_./ _)" [0, 0, 10] 10) + "_Bleast" :: "id => 'a set => bool => 'a" ("(3LEAST _:_./ _)" [0, 0, 10] 10) + syntax (HOL) "_Ball" :: "pttrn => 'a set => bool => bool" ("(3! _:_./ _)" [0, 0, 10] 10) @@ -86,6 +88,8 @@ "INT x:A. B" == "INTER A (%x. B)" "ALL x:A. P" == "Ball A (%x. P)" "EX x:A. P" == "Bex A (%x. P)" + "LEAST x:A. P" => "LEAST x. x:A & P" + syntax (output) "_setle" :: "'a set => 'a set => bool" ("op <=") @@ -108,6 +112,7 @@ Inter :: "'a set set => 'a set" ("\_" [90] 90) "_Ball" :: "pttrn => 'a set => bool => bool" ("(3\_\_./ _)" [0, 0, 10] 10) "_Bex" :: "pttrn => 'a set => bool => bool" ("(3\_\_./ _)" [0, 0, 10] 10) + "_Bleast" :: "id => 'a set => bool => 'a" ("(3LEAST_\_./ _)" [0, 0, 10] 10) syntax (HTML output) "_setle" :: "'a set => 'a set => bool" ("op \")