Minor
authorCezary Kaliszyk <kaliszyk@in.tum.de>
Sat, 12 Dec 2009 09:27:06 +0100
changeset 729 8d5408322de5
parent 728 0015159fee96
child 732 33cd648df179
Minor
Quot/Examples/FSet3.thy
--- a/Quot/Examples/FSet3.thy	Sat Dec 12 05:12:50 2009 +0100
+++ b/Quot/Examples/FSet3.thy	Sat Dec 12 09:27:06 2009 +0100
@@ -34,11 +34,11 @@
 
 
 lemma no_mem_nil: 
-  "(\<forall>a. \<not>(a \<in> set A)) = (A = [])"
+  "(\<forall>a. a \<notin> set A) = (A = [])"
 by (induct A) (auto)
 
 lemma none_mem_nil: 
-  "(\<forall>a. \<not>(a \<in> set A)) = (A \<approx> [])"
+  "(\<forall>a. a \<notin> set A) = (A \<approx> [])"
 by simp
 
 lemma mem_cons: 
@@ -235,7 +235,7 @@
   as "delete_raw"
 
 quotient_def
-  "funion :: 'a fset \<Rightarrow> 'a fset \<Rightarrow> 'a fset" ("_ \<in>f _" [50, 51] 50)
+  "funion :: 'a fset \<Rightarrow> 'a fset \<Rightarrow> 'a fset" ("_ \<union>f _" [50, 51] 50)
   as "op @"
 
 quotient_def
@@ -267,6 +267,8 @@
   MEM x [] = F
   MEM x (h::t) = (x=h) \/ MEM x t *)
 thm none_mem_nil
+(*lemma "(\<forall>a. a \<notin>f A) = (A = fempty)"*)
+
 thm mem_cons
 thm finite_set_raw_strong_cases
 thm card_raw.simps