converted theory "set" to Isar and added some SET-VAR examples
authorpaulson
Thu, 14 Mar 2002 16:48:34 +0100
changeset 13058 ad6106d7b4bb
parent 13057 805de10ca485
child 13059 d78d2089e163
converted theory "set" to Isar and added some SET-VAR examples
src/HOL/ex/set.ML
src/HOL/ex/set.thy
--- a/src/HOL/ex/set.ML	Thu Mar 14 16:00:29 2002 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,123 +0,0 @@
-(*  Title:      HOL/ex/set.ML
-    ID:         $Id$
-    Author:     Tobias Nipkow, Cambridge University Computer Laboratory
-    Copyright   1991  University of Cambridge
-
-Cantor's Theorem; the Schroeder-Berstein Theorem.  
-*)
-
-(*These two are cited in Benzmueller and Kohlhase's system description of LEO,
-  CADE-15, 1998 (page 139-143) as theorems LEO could not prove.*)
-
-Goal "(X = Y Un Z) = (Y<=X & Z<=X & (ALL V. Y<=V & Z<=V --> X<=V))";
-by (Blast_tac 1);
-qed "";
-
-Goal "(X = Y Int Z) = (X<=Y & X<=Z & (ALL V. V<=Y & V<=Z --> V<=X))";
-by (Blast_tac 1);
-qed "";
-
-(*trivial example of term synthesis: apparently hard for some provers!*)
-Goal "a ~= b ==> a:?X & b ~: ?X";
-by (Blast_tac 1);
-qed "";
-
-(** Examples for the Blast_tac paper **)
-
-(*Union-image, called Un_Union_image on equalities.ML*)
-Goal "(UN x:C. f(x) Un g(x)) = Union(f`C)  Un  Union(g`C)";
-by (Blast_tac 1);
-qed "";
-
-(*Inter-image, called Int_Inter_image on equalities.ML*)
-Goal "(INT x:C. f(x) Int g(x)) = Inter(f`C) Int Inter(g`C)";
-by (Blast_tac 1);
-qed "";
-
-(*Singleton I.  Nice demonstration of blast_tac--and its limitations*)
-Goal "!!S::'a set set. ALL x:S. ALL y:S. x<=y ==> EX z. S <= {z}";
-(*for some unfathomable reason, UNIV_I increases the search space greatly*)
-by (blast_tac (claset() delrules [UNIV_I]) 1);
-qed "";
-
-(*Singleton II.  variant of the benchmark above*)
-Goal "ALL x:S. Union(S) <= x ==> EX z. S <= {z}";
-by (blast_tac (claset() delrules [UNIV_I]) 1);
-(*just Blast_tac takes 5 seconds instead of 1*)
-qed "";
-
-(*** A unique fixpoint theorem --- fast/best/meson all fail ***)
-
-Goal "EX! x. f(g(x))=x ==> EX! y. g(f(y))=y";
-by (EVERY1[etac ex1E, rtac ex1I, etac arg_cong,
-          rtac subst, atac, etac allE, rtac arg_cong, etac mp, etac arg_cong]);
-qed "";
-
-
-(*** Cantor's Theorem: There is no surjection from a set to its powerset. ***)
-
-Goal "~ (EX f:: 'a=>'a set. ALL S. EX x. f(x) = S)";
-(*requires best-first search because it is undirectional*)
-by (Best_tac 1);
-qed "cantor1";
-
-(*This form displays the diagonal term*)
-Goal "ALL f:: 'a=>'a set. ALL x. f(x) ~= ?S(f)";
-by (Best_tac 1);
-uresult();
-
-(*This form exploits the set constructs*)
-Goal "?S ~: range(f :: 'a=>'a set)";
-by (rtac notI 1);
-by (etac rangeE 1);
-by (etac equalityCE 1);
-by (dtac CollectD 1);
-by (contr_tac 1);
-by (swap_res_tac [CollectI] 1);
-by (assume_tac 1);
-
-choplev 0;
-by (Best_tac 1);
-qed "";
-
-
-(*** The Schroeder-Berstein Theorem ***)
-
-Goal "[| -(f`X) = g`(-X);  f(a)=g(b);  a:X |] ==> b:X";
-by (Blast_tac 1);
-qed "disj_lemma";
-
-Goal "-(f`X) = g`(-X) ==> surj(%z. if z:X then f(z) else g(z))";
-by (asm_simp_tac (simpset() addsimps [surj_def]) 1);
-by (Blast_tac 1);
-qed "surj_if_then_else";
-
-Goalw [inj_on_def]
-     "[| inj_on f X;  inj_on g (-X);  -(f`X) = g`(-X); \
-\        h = (%z. if z:X then f(z) else g(z)) |]       \
-\     ==> inj(h) & surj(h)";
-by (asm_simp_tac (simpset() addsimps [surj_if_then_else]) 1);
-by (blast_tac (claset() addDs [disj_lemma, sym]) 1);
-qed "bij_if_then_else";
-
-Goal "EX X. X = - (g`(- (f`X)))";
-by (rtac exI 1);
-by (rtac lfp_unfold 1);
-by (REPEAT (ares_tac [monoI, image_mono, Compl_anti_mono] 1));
-qed "decomposition";
-
-val [injf,injg] = goal (the_context ())
-   "[| inj (f:: 'a=>'b);  inj (g:: 'b=>'a) |] \
-\   ==> EX h:: 'a=>'b. inj(h) & surj(h)";
-by (rtac (decomposition RS exE) 1);
-by (rtac exI 1);
-by (rtac bij_if_then_else 1);
-by (rtac refl 4);
-by (rtac inj_on_inv 2);
-by (rtac ([subset_UNIV, injf] MRS subset_inj_on) 1);
-  (**tricky variable instantiations!**)
-by (EVERY1 [etac ssubst, stac double_complement, rtac subsetI,
-            etac imageE, etac ssubst, rtac rangeI]);
-by (EVERY1 [etac ssubst, stac double_complement, 
-            rtac (injg RS inv_image_comp RS sym)]);
-qed "schroeder_bernstein";
--- a/src/HOL/ex/set.thy	Thu Mar 14 16:00:29 2002 +0100
+++ b/src/HOL/ex/set.thy	Thu Mar 14 16:48:34 2002 +0100
@@ -1,4 +1,177 @@
+(*  Title:      HOL/ex/set.thy
+    ID:         $Id$
+    Author:     Tobias Nipkow and Lawrence C Paulson
+    Copyright   1991  University of Cambridge
+
+Set Theory examples: Cantor's Theorem, Schroeder-Berstein Theorem, etc.
+*)
 
 theory set = Main:
 
+text{*These two are cited in Benzmueller and Kohlhase's system description 
+of LEO, CADE-15, 1998 (pages 139-143) as theorems LEO could not prove.*}
+
+lemma "(X = Y Un Z) = (Y<=X & Z<=X & (ALL V. Y<=V & Z<=V --> X<=V))"
+by blast
+
+lemma "(X = Y Int Z) = (X<=Y & X<=Z & (ALL V. V<=Y & V<=Z --> V<=X))"
+by blast
+
+text{*trivial example of term synthesis: apparently hard for some provers!*}
+lemma "a ~= b ==> a:?X & b ~: ?X"
+by blast
+
+(** Examples for the Blast_tac paper **)
+
+text{*Union-image, called Un_Union_image on equalities.ML*}
+lemma "(UN x:C. f(x) Un g(x)) = Union(f`C)  Un  Union(g`C)"
+by blast
+
+text{*Inter-image, called Int_Inter_image on equalities.ML*}
+lemma "(INT x:C. f(x) Int g(x)) = Inter(f`C) Int Inter(g`C)"
+by blast
+
+text{*Singleton I.  Nice demonstration of blast_tac--and its limitations.
+For some unfathomable reason, UNIV_I increases the search space greatly*}
+lemma "!!S::'a set set. ALL x:S. ALL y:S. x<=y ==> EX z. S <= {z}"
+by (blast del: UNIV_I)
+
+text{*Singleton II.  variant of the benchmark above*}
+lemma "ALL x:S. Union(S) <= x ==> EX z. S <= {z}"
+by (blast del: UNIV_I)
+
+text{* A unique fixpoint theorem --- fast/best/meson all fail *}
+
+lemma "EX! x. f(g(x))=x ==> EX! y. g(f(y))=y"
+apply (erule ex1E, rule ex1I, erule arg_cong)
+apply (rule subst, assumption, erule allE, rule arg_cong, erule mp) 
+apply (erule arg_cong) 
+done
+
+
+
+text{* Cantor's Theorem: There is no surjection from a set to its powerset. *}
+
+text{*requires best-first search because it is undirectional*}
+lemma cantor1: "~ (EX f:: 'a=>'a set. ALL S. EX x. f(x) = S)"
+by best
+
+text{*This form displays the diagonal term*}
+lemma "ALL f:: 'a=>'a set. ALL x. f(x) ~= ?S(f)"
+by best
+
+text{*This form exploits the set constructs*}
+lemma "?S ~: range(f :: 'a=>'a set)"
+by (rule notI, erule rangeE, best)  
+
+text{*Or just this!*}
+lemma "?S ~: range(f :: 'a=>'a set)"
+by best
+
+text{* The Schroeder-Berstein Theorem *}
+
+lemma disj_lemma: "[| -(f`X) = g`(-X);  f(a)=g(b);  a:X |] ==> b:X"
+by blast
+
+lemma surj_if_then_else:
+     "-(f`X) = g`(-X) ==> surj(%z. if z:X then f(z) else g(z))"
+by (simp add: surj_def, blast)
+
+lemma bij_if_then_else: 
+     "[| inj_on f X;  inj_on g (-X);  -(f`X) = g`(-X);  
+         h = (%z. if z:X then f(z) else g(z)) |]        
+      ==> inj(h) & surj(h)"
+apply (unfold inj_on_def)
+apply (simp add: surj_if_then_else)
+apply (blast dest: disj_lemma sym)
+done
+
+lemma decomposition: "EX X. X = - (g`(- (f`X)))"
+apply (rule exI)
+apply (rule lfp_unfold)
+apply (rule monoI, blast) 
+done
+
+text{*Schroeder-Bernstein Theorem*}
+lemma "[| inj (f:: 'a=>'b);  inj (g:: 'b=>'a) |]  
+       ==> EX h:: 'a=>'b. inj(h) & surj(h)"
+apply (rule decomposition [THEN exE])
+apply (rule exI)
+apply (rule bij_if_then_else)
+   apply (rule_tac [4] refl)
+  apply (rule_tac [2] inj_on_inv)
+  apply (erule subset_inj_on [OF subset_UNIV]) 
+  txt{*tricky variable instantiations!*}
+ apply (erule ssubst, subst double_complement)
+ apply (rule subsetI, erule imageE, erule ssubst, rule rangeI) 
+apply (erule ssubst, subst double_complement, erule inv_image_comp [symmetric])
+done
+
+
+text{*Set variable instantiation examples from 
+W. W. Bledsoe and Guohui Feng, SET-VAR.
+JAR 11 (3), 1993, pages 293-314.
+
+Isabelle can prove the easy examples without any special mechanisms, but it
+can't prove the hard ones.
+*}
+
+text{*Example 1, page 295.*}
+lemma "(EX A. (ALL x:A. x <= (0::int)))"
+by force 
+
+text{*Example 2*}
+lemma "D : F --> (EX G. (ALL A:G. EX B:F. A <= B))";
+by force 
+
+text{*Example 3*}
+lemma "P(a) --> (EX A. (ALL x:A. P(x)) & (EX y. y:A))";
+by force 
+
+text{*Example 4*}
+lemma "a<b & b<(c::int) --> (EX A. a~:A & b:A & c~: A)"
+by force 
+
+text{*Example 5, page 298.*}
+lemma "P(f(b)) --> (EX s A. (ALL x:A. P(x)) & f(s):A)";
+by force 
+
+text{*Example 6*}
+lemma "P(f(b)) --> (EX s A. (ALL x:A. P(x)) & f(s):A)";
+by force 
+
+text{*Example 7*}
+lemma "EX A. a ~: A"
+by force 
+
+text{*Example 8*}
+lemma "(ALL u v. u < (0::int) --> u ~= abs v) --> (EX A::int set. (ALL y. abs y ~: A) & -2 : A)"
+by force  text{*not blast, which can't simplify -2<0*}
+
+text{*Example 9 omitted (requires the reals)*}
+
+text{*The paper has no Example 10!*}
+
+text{*Example 11: needs a hint*}
+lemma "(ALL A. 0:A & (ALL x:A. Suc(x):A) --> n:A) & 
+       P(0) & (ALL x. P(x) --> P(Suc(x))) --> P(n)"
+apply clarify
+apply (drule_tac x="{x. P x}" in spec)
+by force  
+
+text{*Example 12*}
+lemma "(ALL A. (0,0):A & (ALL x y. (x,y):A --> (Suc(x),Suc(y)):A) --> (n,m):A)
+       & P(n) --> P(m)"
+by auto 
+
+text{*Example EO1: typo in article, and with the obvious fix it seems
+      to require arithmetic reasoning.*}
+lemma "(ALL x. (EX u. x=2*u) = (~(EX v. Suc x = 2*v))) --> 
+       (EX A. ALL x. (x : A) = (Suc x ~: A))"
+apply clarify 
+apply (rule_tac x="{x. EX u. x = 2*u}" in exI, auto) 
+apply (case_tac v, auto)
+apply (drule_tac x="Suc v" and P="%x. ?a(x) ~= ?b(x)" in spec, force) 
+done
+
 end