# HG changeset patch # User paulson # Date 859195703 -3600 # Node ID c07d6bc56cc297762068582bc7be6ba5e8942416 # Parent 9b47fc57ab7a4c845ee3e2620d00ed38ee4438ee Deleted needless parentheses diff -r 9b47fc57ab7a -r c07d6bc56cc2 src/ZF/func.ML --- a/src/ZF/func.ML Mon Mar 24 10:27:28 1997 +0100 +++ b/src/ZF/func.ML Mon Mar 24 10:28:23 1997 +0100 @@ -34,7 +34,7 @@ qed "fun_is_rel"; goal thy "!!f. [| f: Pi(A,B); a:A |] ==> EX! y. : f"; -by (fast_tac ((!claset) addSDs [Pi_iff_old RS iffD1]) 1); +by (fast_tac (!claset addSDs [Pi_iff_old RS iffD1]) 1); qed "fun_unique_Pair"; val prems = goalw thy [Pi_def] @@ -94,7 +94,7 @@ goal thy "!!f. [| f: Pi(A,B); c: f |] ==> EX x:A. c = "; by (forward_tac [fun_is_rel] 1); -by (fast_tac ((!claset) addDs [apply_equality]) 1); +by (fast_tac (!claset addDs [apply_equality]) 1); qed "Pi_memberD"; goal thy "!!f. [| f: Pi(A,B); a:A |] ==> : f"; @@ -117,8 +117,8 @@ val [major] = goal thy "f: Pi(A,B) ==> : f <-> a:A & f`a = b"; by (cut_facts_tac [major RS fun_is_rel] 1); -by (fast_tac ((!claset) addSIs [major RS apply_Pair, - major RSN (2,apply_equality)]) 1); +by (fast_tac (!claset addSIs [major RS apply_Pair, + major RSN (2,apply_equality)]) 1); qed "apply_iff"; (*Refining one Pi type to another*) @@ -126,7 +126,7 @@ "[| f: Pi(A,C); !!x. x:A ==> f`x : B(x) |] ==> f : Pi(A,B)"; by (cut_facts_tac [pi_prem] 1); by (asm_full_simp_tac (FOL_ss addsimps [Pi_iff]) 1); -by (fast_tac ((!claset) addIs prems addSDs [pi_prem RS Pi_memberD]) 1); +by (fast_tac (!claset addIs prems addSDs [pi_prem RS Pi_memberD]) 1); qed "Pi_type"; @@ -169,7 +169,7 @@ val prems = goalw thy [lam_def, Pi_def, function_def] "[| !!x. x:A ==> b(x): B(x) |] ==> (lam x:A.b(x)) : Pi(A,B)"; -by (fast_tac ((!claset) addIs prems) 1); +by (fast_tac (!claset addIs prems) 1); qed "lam_type"; goal thy "(lam x:A.b(x)) : A -> {b(x). x:A}"; @@ -259,7 +259,7 @@ goalw thy [restrict_def,lam_def] "!!f A. [| f: Pi(C,B); A<=C |] ==> restrict(f,A) <= f"; -by (fast_tac ((!claset) addIs [apply_Pair]) 1); +by (fast_tac (!claset addIs [apply_Pair]) 1); qed "restrict_subset"; val prems = goalw thy [restrict_def] @@ -310,7 +310,7 @@ "!!S. [| ALL x:S. function(x); \ \ ALL x:S. ALL y:S. x<=y | y<=x |] ==> \ \ function(Union(S))"; -by (fast_tac ((!claset) addSDs [bspec RS bspec]) 1); +by (fast_tac (!claset addSDs [bspec RS bspec]) 1); qed "function_Union"; goalw thy [Pi_def] @@ -384,7 +384,7 @@ goal thy "!!f A B. [| f: A->B; c~:A; b: B |] ==> cons(,f) : cons(c,A) -> B"; -by (fast_tac ((!claset) addEs [fun_extend RS fun_weaken_type]) 1); +by (fast_tac (!claset addEs [fun_extend RS fun_weaken_type]) 1); qed "fun_extend3"; goal thy "!!f A B. [| f: A->B; a:A; c~:A |] ==> cons(,f)`a = f`a"; @@ -406,10 +406,10 @@ goal thy "!!c. c ~: A ==> cons(c,A) -> B = (UN f: A->B. UN b:B. {cons(, f)})"; by (rtac equalityI 1); -by (safe_tac ((!claset) addSEs [fun_extend3])); +by (safe_tac (!claset addSEs [fun_extend3])); (*Inclusion of left into right*) by (subgoal_tac "restrict(x, A) : A -> B" 1); -by (fast_tac ((!claset) addEs [restrict_type2]) 2); +by (fast_tac (!claset addEs [restrict_type2]) 2); by (rtac UN_I 1 THEN assume_tac 1); by (rtac (apply_funtype RS UN_I) 1 THEN REPEAT (ares_tac [consI1] 1)); by (Simp_tac 1);