equal
deleted
inserted
replaced
25 subset :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" where |
25 subset :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" where |
26 "subset = op \<subseteq>" |
26 "subset = op \<subseteq>" |
27 |
27 |
28 lemmas [symmetric, code inline] = subset_def |
28 lemmas [symmetric, code inline] = subset_def |
29 |
29 |
|
30 definition |
|
31 strict_subset :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" where |
|
32 "strict_subset = op \<subset>" |
|
33 |
|
34 lemmas [symmetric, code inline] = strict_subset_def |
|
35 |
30 lemma [code target: Set]: |
36 lemma [code target: Set]: |
31 "A = B \<longleftrightarrow> A \<subseteq> B \<and> B \<subseteq> A" |
37 "A = B \<longleftrightarrow> A \<subseteq> B \<and> B \<subseteq> A" |
32 by blast |
38 by blast |
33 |
39 |
34 lemma [code func]: |
40 lemma [code func]: |
|
41 "(A\<Colon>'a\<Colon>eq set) = B \<longleftrightarrow> A \<subseteq> B \<and> B \<subseteq> A" |
|
42 by blast |
|
43 |
|
44 lemma [code func]: |
35 "subset A B \<longleftrightarrow> (\<forall>x\<in>A. x \<in> B)" |
45 "subset A B \<longleftrightarrow> (\<forall>x\<in>A. x \<in> B)" |
36 unfolding subset_def Set.subset_def .. |
46 unfolding subset_def Set.subset_def .. |
|
47 |
|
48 lemma [code func]: |
|
49 "strict_subset A B \<longleftrightarrow> subset A B \<and> A \<noteq> B" |
|
50 unfolding subset_def strict_subset_def by blast |
37 |
51 |
38 lemma [code]: |
52 lemma [code]: |
39 "a \<in> A \<longleftrightarrow> (\<exists>x\<in>A. x = a)" |
53 "a \<in> A \<longleftrightarrow> (\<exists>x\<in>A. x = a)" |
40 unfolding bex_triv_one_point1 .. |
54 unfolding bex_triv_one_point1 .. |
41 |
55 |