src/ZF/mono.ML
author nipkow
Thu, 26 Nov 1998 12:18:08 +0100
changeset 5974 6acf3ff0f486
parent 5325 f7a5e06adea1
child 6053 8a1059aa01f0
permissions -rw-r--r--
Added filter_prems_tac
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 811
diff changeset
     1
(*  Title:      ZF/mono
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     2
    ID:         $Id$
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 811
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     4
    Copyright   1993  University of Cambridge
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     5
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     6
Monotonicity of various operations (for lattice properties see subset.ML)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     7
*)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     8
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
     9
open mono;
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
    10
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    11
(** Replacement, in its various formulations **)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    12
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    13
(*Not easy to express monotonicity in P, since any "bigger" predicate
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    14
  would have to be single-valued*)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    15
Goal "A<=B ==> Replace(A,P) <= Replace(B,P)";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3890
diff changeset
    16
by (blast_tac (claset() addSEs [ReplaceE]) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    17
qed "Replace_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    18
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    19
Goal "A<=B ==> {f(x). x:A} <= {f(x). x:B}";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    20
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    21
qed "RepFun_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    22
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    23
Goal "A<=B ==> Pow(A) <= Pow(B)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    24
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    25
qed "Pow_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    26
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    27
Goal "A<=B ==> Union(A) <= Union(B)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    28
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    29
qed "Union_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    30
5325
f7a5e06adea1 Yet more removal of "goal" commands, especially "goal ZF.thy", so ZF.thy
paulson
parents: 5137
diff changeset
    31
val prems = Goal
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    32
    "[| A<=C;  !!x. x:A ==> B(x)<=D(x) \
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    33
\    |] ==> (UN x:A. B(x)) <= (UN x:C. D(x))";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3890
diff changeset
    34
by (blast_tac (claset() addIs (prems RL [subsetD])) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    35
qed "UN_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    36
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    37
(*Intersection is ANTI-monotonic.  There are TWO premises! *)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    38
Goal "[| A<=B;  a:A |] ==> Inter(B) <= Inter(A)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    39
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    40
qed "Inter_anti_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    41
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    42
Goal "C<=D ==> cons(a,C) <= cons(a,D)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    43
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    44
qed "cons_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    45
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    46
Goal "[| A<=C;  B<=D |] ==> A Un B <= C Un D";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    47
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    48
qed "Un_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    49
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    50
Goal "[| A<=C;  B<=D |] ==> A Int B <= C Int D";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    51
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    52
qed "Int_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    53
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    54
Goal "[| A<=C;  D<=B |] ==> A-B <= C-D";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    55
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    56
qed "Diff_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    57
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    58
(** Standard products, sums and function spaces **)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    59
5325
f7a5e06adea1 Yet more removal of "goal" commands, especially "goal ZF.thy", so ZF.thy
paulson
parents: 5137
diff changeset
    60
Goal "[| A<=C;  ALL x:A. B(x) <= D(x) |] ==> Sigma(A,B) <= Sigma(C,D)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    61
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    62
qed "Sigma_mono_lemma";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    63
val Sigma_mono = ballI RSN (2,Sigma_mono_lemma);
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    64
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    65
Goalw sum_defs "[| A<=C;  B<=D |] ==> A+B <= C+D";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    66
by (REPEAT (ares_tac [subset_refl,Un_mono,Sigma_mono] 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    67
qed "sum_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    68
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    69
(*Note that B->A and C->A are typically disjoint!*)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    70
Goal "B<=C ==> A->B <= A->C";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3890
diff changeset
    71
by (blast_tac (claset() addIs [lam_type] addEs [Pi_lamE]) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    72
qed "Pi_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    73
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    74
Goalw [lam_def] "A<=B ==> Lambda(A,c) <= Lambda(B,c)";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    75
by (etac RepFun_mono 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    76
qed "lam_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    77
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    78
(** Quine-inspired ordered pairs, products, injections and sums **)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    79
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    80
Goalw [QPair_def] "[| a<=c;  b<=d |] ==> <a;b> <= <c;d>";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    81
by (REPEAT (ares_tac [sum_mono] 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    82
qed "QPair_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    83
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    84
Goal "[| A<=C;  ALL x:A. B(x) <= D(x) |] ==>  \
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    85
\                          QSigma(A,B) <= QSigma(C,D)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    86
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    87
qed "QSigma_mono_lemma";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    88
val QSigma_mono = ballI RSN (2,QSigma_mono_lemma);
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    89
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    90
Goalw [QInl_def] "a<=b ==> QInl(a) <= QInl(b)";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    91
by (REPEAT (ares_tac [subset_refl RS QPair_mono] 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    92
qed "QInl_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    93
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    94
Goalw [QInr_def] "a<=b ==> QInr(a) <= QInr(b)";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    95
by (REPEAT (ares_tac [subset_refl RS QPair_mono] 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
    96
qed "QInr_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    97
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
    98
Goal "[| A<=C;  B<=D |] ==> A <+> B <= C <+> D";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
    99
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   100
qed "qsum_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   101
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   102
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   103
(** Converse, domain, range, field **)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   104
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
   105
Goal "r<=s ==> converse(r) <= converse(s)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
   106
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   107
qed "converse_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   108
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
   109
Goal "r<=s ==> domain(r)<=domain(s)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
   110
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   111
qed "domain_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   112
811
9bac814082e4 Used bind_thm to store domain_rel_subset and range_rel_subset
lcp
parents: 760
diff changeset
   113
bind_thm ("domain_rel_subset", [domain_mono, domain_subset] MRS subset_trans);
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   114
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
   115
Goal "r<=s ==> range(r)<=range(s)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
   116
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   117
qed "range_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   118
811
9bac814082e4 Used bind_thm to store domain_rel_subset and range_rel_subset
lcp
parents: 760
diff changeset
   119
bind_thm ("range_rel_subset", [range_mono, range_subset] MRS subset_trans);
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   120
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
   121
Goal "r<=s ==> field(r)<=field(s)";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
   122
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   123
qed "field_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   124
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
   125
Goal "r <= A*A ==> field(r) <= A";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   126
by (etac (field_mono RS subset_trans) 1);
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
   127
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   128
qed "field_rel_subset";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   129
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   130
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   131
(** Images **)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   132
5325
f7a5e06adea1 Yet more removal of "goal" commands, especially "goal ZF.thy", so ZF.thy
paulson
parents: 5137
diff changeset
   133
val [prem1,prem2] = Goal
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   134
    "[| !! x y. <x,y>:r ==> <x,y>:s;  A<=B |] ==> r``A <= s``B";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3890
diff changeset
   135
by (blast_tac (claset() addIs [prem1, prem2 RS subsetD]) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   136
qed "image_pair_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   137
5325
f7a5e06adea1 Yet more removal of "goal" commands, especially "goal ZF.thy", so ZF.thy
paulson
parents: 5137
diff changeset
   138
val [prem1,prem2] = Goal
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   139
    "[| !! x y. <x,y>:r ==> <x,y>:s;  A<=B |] ==> r-``A <= s-``B";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3890
diff changeset
   140
by (blast_tac (claset() addIs [prem1, prem2 RS subsetD]) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   141
qed "vimage_pair_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   142
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
   143
Goal "[| r<=s;  A<=B |] ==> r``A <= s``B";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
   144
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   145
qed "image_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   146
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
   147
Goal "[| r<=s;  A<=B |] ==> r-``A <= s-``B";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
   148
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   149
qed "vimage_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   150
5325
f7a5e06adea1 Yet more removal of "goal" commands, especially "goal ZF.thy", so ZF.thy
paulson
parents: 5137
diff changeset
   151
val [sub,PQimp] = Goal
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   152
    "[| A<=B;  !!x. x:A ==> P(x) --> Q(x) |] ==> Collect(A,P) <= Collect(B,Q)";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3890
diff changeset
   153
by (blast_tac (claset() addIs [sub RS subsetD, PQimp RS mp]) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   154
qed "Collect_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   155
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   156
(** Monotonicity of implications -- some could go to FOL **)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   157
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5067
diff changeset
   158
Goal "A<=B ==> x:A --> x:B";
2925
b0ae2e13db93 Using Blast_tac
paulson
parents: 2803
diff changeset
   159
by (Blast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   160
qed "in_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   161
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   162
goal IFOL.thy "!!P1 P2 Q1 Q2. [| P1-->Q1; P2-->Q2 |] ==> (P1&P2) --> (Q1&Q2)";
2602
5ac837d98a85 Renamed structure Int (intuitionistic prover) to IntPr
paulson
parents: 2469
diff changeset
   163
by (IntPr.fast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   164
qed "conj_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   165
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   166
goal IFOL.thy "!!P1 P2 Q1 Q2. [| P1-->Q1; P2-->Q2 |] ==> (P1|P2) --> (Q1|Q2)";
2602
5ac837d98a85 Renamed structure Int (intuitionistic prover) to IntPr
paulson
parents: 2469
diff changeset
   167
by (IntPr.fast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   168
qed "disj_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   169
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   170
goal IFOL.thy "!!P1 P2 Q1 Q2.[| Q1-->P1; P2-->Q2 |] ==> (P1-->P2)-->(Q1-->Q2)";
2602
5ac837d98a85 Renamed structure Int (intuitionistic prover) to IntPr
paulson
parents: 2469
diff changeset
   171
by (IntPr.fast_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   172
qed "imp_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   173
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   174
goal IFOL.thy "P-->P";
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   175
by (rtac impI 1);
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   176
by (assume_tac 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   177
qed "imp_refl";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   178
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   179
val [PQimp] = goal IFOL.thy
3840
e0baea4d485a fixed dots;
wenzelm
parents: 3015
diff changeset
   180
    "[| !!x. P(x) --> Q(x) |] ==> (EX x. P(x)) --> (EX x. Q(x))";
2803
734fc343ec2a Conducted the IFOL proofs using intuitionistic tools
paulson
parents: 2602
diff changeset
   181
by IntPr.safe_tac;
3015
65778b9d865f Ran expandshort
paulson
parents: 2925
diff changeset
   182
by (etac (PQimp RS mp RS exI) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   183
qed "ex_mono";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   184
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   185
val [PQimp] = goal IFOL.thy
3840
e0baea4d485a fixed dots;
wenzelm
parents: 3015
diff changeset
   186
    "[| !!x. P(x) --> Q(x) |] ==> (ALL x. P(x)) --> (ALL x. Q(x))";
2803
734fc343ec2a Conducted the IFOL proofs using intuitionistic tools
paulson
parents: 2602
diff changeset
   187
by IntPr.safe_tac;
3015
65778b9d865f Ran expandshort
paulson
parents: 2925
diff changeset
   188
by (etac (spec RS (PQimp RS mp)) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 744
diff changeset
   189
qed "all_mono";
516
1957113f0d7d installation of new inductive/datatype sections
lcp
parents: 485
diff changeset
   190
1957113f0d7d installation of new inductive/datatype sections
lcp
parents: 485
diff changeset
   191
(*Used in intr_elim.ML and in individual datatype definitions*)
1957113f0d7d installation of new inductive/datatype sections
lcp
parents: 485
diff changeset
   192
val basic_monos = [subset_refl, imp_refl, disj_mono, conj_mono, 
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 811
diff changeset
   193
                   ex_mono, Collect_mono, Part_mono, in_mono];
516
1957113f0d7d installation of new inductive/datatype sections
lcp
parents: 485
diff changeset
   194