src/ZF/QPair.thy
author wenzelm
Sun, 17 Dec 2023 21:12:18 +0100
changeset 79270 90c5aadcc4b2
parent 76215 a642599ffdea
permissions -rw-r--r--
more robust norm_proof: turn env into instantiation, based on visible statement;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
35762
af3ff2ba4c54 removed old CVS Ids;
wenzelm
parents: 24893
diff changeset
     1
(*  Title:      ZF/QPair.thy
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
     2
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     3
    Copyright   1993  University of Cambridge
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     4
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
     5
Many proofs are borrowed from pair.thy and sum.thy
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
     6
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
     7
Do we EVER have rank(a) < rank(<a;b>) ?  Perhaps if the latter rank
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
     8
is not a limit ordinal?
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     9
*)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    10
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
    11
section\<open>Quine-Inspired Ordered Pairs and Disjoint Sums\<close>
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13285
diff changeset
    12
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 14854
diff changeset
    13
theory QPair imports Sum func begin
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    14
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
    15
text\<open>For non-well-founded data
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13285
diff changeset
    16
structures in ZF.  Does not precisely follow Quine's construction.  Thanks
c9cfe1638bf2 improved presentation markup
paulson
parents: 13285
diff changeset
    17
to Thomas Forster for suggesting this approach!
c9cfe1638bf2 improved presentation markup
paulson
parents: 13285
diff changeset
    18
c9cfe1638bf2 improved presentation markup
paulson
parents: 13285
diff changeset
    19
W. V. Quine, On Ordered Pairs and Relations, in Selected Logic Papers,
c9cfe1638bf2 improved presentation markup
paulson
parents: 13285
diff changeset
    20
1966.
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
    21
\<close>
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13285
diff changeset
    22
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    23
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    24
  QPair     :: "[i, i] \<Rightarrow> i"                      (\<open><(_;/ _)>\<close>)  where
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    25
    "<a;b> \<equiv> a+b"
3923
c257b82a1200 global;
wenzelm
parents: 2469
diff changeset
    26
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    27
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    28
  qfst :: "i \<Rightarrow> i"  where
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    29
    "qfst(p) \<equiv> THE a. \<exists>b. p=<a;b>"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    30
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    31
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    32
  qsnd :: "i \<Rightarrow> i"  where
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    33
    "qsnd(p) \<equiv> THE b. \<exists>a. p=<a;b>"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    34
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    35
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    36
  qsplit    :: "[[i, i] \<Rightarrow> 'a, i] \<Rightarrow> 'a::{}"  (*for pattern-matching*)  where
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    37
    "qsplit(c,p) \<equiv> c(qfst(p), qsnd(p))"
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    38
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    39
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    40
  qconverse :: "i \<Rightarrow> i"  where
76214
0c18df79b1c8 more modernisation of syntax
paulson <lp15@cam.ac.uk>
parents: 76213
diff changeset
    41
    "qconverse(r) \<equiv> {z. w \<in> r, \<exists>x y. w=<x;y> \<and> z=<y;x>}"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    42
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    43
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    44
  QSigma    :: "[i, i \<Rightarrow> i] \<Rightarrow> i"  where
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    45
    "QSigma(A,B)  \<equiv>  \<Union>x\<in>A. \<Union>y\<in>B(x). {<x;y>}"
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    46
929
137035296ad6 Moved declarations of @QSUM and <*> to a syntax section.
lcp
parents: 753
diff changeset
    47
syntax
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    48
  "_QSUM"   :: "[idt, i, i] \<Rightarrow> i"               (\<open>(3QSUM _ \<in> _./ _)\<close> 10)
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    49
translations
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    50
  "QSUM x \<in> A. B" => "CONST QSigma(A, \<lambda>x. B)"
22808
a7daa74e2980 eliminated unnamed infixes, tuned syntax;
wenzelm
parents: 17782
diff changeset
    51
a7daa74e2980 eliminated unnamed infixes, tuned syntax;
wenzelm
parents: 17782
diff changeset
    52
abbreviation
69587
53982d5ec0bb isabelle update -u mixfix_cartouches;
wenzelm
parents: 60770
diff changeset
    53
  qprod  (infixr \<open><*>\<close> 80) where
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    54
  "A <*> B \<equiv> QSigma(A, \<lambda>_. B)"
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    55
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    56
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    57
  qsum    :: "[i,i]\<Rightarrow>i"                         (infixr \<open><+>\<close> 65)  where
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    58
    "A <+> B      \<equiv> ({0} <*> A) \<union> ({1} <*> B)"
3923
c257b82a1200 global;
wenzelm
parents: 2469
diff changeset
    59
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    60
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    61
  QInl :: "i\<Rightarrow>i"  where
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    62
    "QInl(a)      \<equiv> <0;a>"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    63
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    64
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    65
  QInr :: "i\<Rightarrow>i"  where
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    66
    "QInr(b)      \<equiv> <1;b>"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    67
24893
b8ef7afe3a6b modernized specifications;
wenzelm
parents: 22808
diff changeset
    68
definition
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    69
  qcase     :: "[i\<Rightarrow>i, i\<Rightarrow>i, i]\<Rightarrow>i"  where
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
    70
    "qcase(c,d)   \<equiv> qsplit(\<lambda>y z. cond(y, d(z), c(z)))"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    71
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    72
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
    73
subsection\<open>Quine ordered pairing\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    74
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    75
(** Lemmas for showing that <a;b> uniquely determines a and b **)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    76
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    77
lemma QPair_empty [simp]: "<0;0> = 0"
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    78
by (simp add: QPair_def)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    79
76214
0c18df79b1c8 more modernisation of syntax
paulson <lp15@cam.ac.uk>
parents: 76213
diff changeset
    80
lemma QPair_iff [simp]: "<a;b> = <c;d> \<longleftrightarrow> a=c \<and> b=d"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    81
apply (simp add: QPair_def)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    82
apply (rule sum_equal_iff)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    83
done
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    84
45602
2a858377c3d2 eliminated obsolete "standard";
wenzelm
parents: 35762
diff changeset
    85
lemmas QPair_inject = QPair_iff [THEN iffD1, THEN conjE, elim!]
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    86
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    87
lemma QPair_inject1: "<a;b> = <c;d> \<Longrightarrow> a=c"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    88
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    89
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    90
lemma QPair_inject2: "<a;b> = <c;d> \<Longrightarrow> b=d"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    91
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    92
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    93
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
    94
subsubsection\<open>QSigma: Disjoint union of a family of sets
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
    95
     Generalizes Cartesian product\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    96
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
    97
lemma QSigmaI [intro!]: "\<lbrakk>a \<in> A;  b \<in> B(a)\<rbrakk> \<Longrightarrow> <a;b> \<in> QSigma(A,B)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    98
by (simp add: QSigma_def)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
    99
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   100
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   101
(** Elimination rules for <a;b>:A*B -- introducing no eigenvariables **)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   102
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   103
lemma QSigmaE [elim!]:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   104
    "\<lbrakk>c \<in> QSigma(A,B);
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   105
        \<And>x y.\<lbrakk>x \<in> A;  y \<in> B(x);  c=<x;y>\<rbrakk> \<Longrightarrow> P
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   106
\<rbrakk> \<Longrightarrow> P"
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   107
by (simp add: QSigma_def, blast)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   108
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   109
lemma QSigmaE2 [elim!]:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   110
    "\<lbrakk><a;b>: QSigma(A,B); \<lbrakk>a \<in> A;  b \<in> B(a)\<rbrakk> \<Longrightarrow> P\<rbrakk> \<Longrightarrow> P"
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   111
by (simp add: QSigma_def)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   112
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   113
lemma QSigmaD1: "<a;b> \<in> QSigma(A,B) \<Longrightarrow> a \<in> A"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   114
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   115
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   116
lemma QSigmaD2: "<a;b> \<in> QSigma(A,B) \<Longrightarrow> b \<in> B(a)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   117
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   118
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   119
lemma QSigma_cong:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   120
    "\<lbrakk>A=A';  \<And>x. x \<in> A' \<Longrightarrow> B(x)=B'(x)\<rbrakk> \<Longrightarrow>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   121
     QSigma(A,B) = QSigma(A',B')"
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   122
by (simp add: QSigma_def)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   123
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   124
lemma QSigma_empty1 [simp]: "QSigma(0,B) = 0"
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   125
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   126
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   127
lemma QSigma_empty2 [simp]: "A <*> 0 = 0"
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   128
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   129
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   130
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
   131
subsubsection\<open>Projections: qfst, qsnd\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   132
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   133
lemma qfst_conv [simp]: "qfst(<a;b>) = a"
13544
895994073bdf various new lemmas for Constructible
paulson
parents: 13534
diff changeset
   134
by (simp add: qfst_def)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   135
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   136
lemma qsnd_conv [simp]: "qsnd(<a;b>) = b"
13544
895994073bdf various new lemmas for Constructible
paulson
parents: 13534
diff changeset
   137
by (simp add: qsnd_def)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   138
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   139
lemma qfst_type [TC]: "p \<in> QSigma(A,B) \<Longrightarrow> qfst(p) \<in> A"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   140
by auto
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   141
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   142
lemma qsnd_type [TC]: "p \<in> QSigma(A,B) \<Longrightarrow> qsnd(p) \<in> B(qfst(p))"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   143
by auto
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   144
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   145
lemma QPair_qfst_qsnd_eq: "a \<in> QSigma(A,B) \<Longrightarrow> <qfst(a); qsnd(a)> = a"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   146
by auto
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   147
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   148
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
   149
subsubsection\<open>Eliminator: qsplit\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   150
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   151
(*A META-equality, so that it applies to higher types as well...*)
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
   152
lemma qsplit [simp]: "qsplit(\<lambda>x y. c(x,y), <a;b>) \<equiv> c(a,b)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   153
by (simp add: qsplit_def)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   154
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   155
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   156
lemma qsplit_type [elim!]:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   157
    "\<lbrakk>p \<in> QSigma(A,B);
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   158
         \<And>x y.\<lbrakk>x \<in> A; y \<in> B(x)\<rbrakk> \<Longrightarrow> c(x,y):C(<x;y>)
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
   159
\<rbrakk> \<Longrightarrow> qsplit(\<lambda>x y. c(x,y), p) \<in> C(p)"
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   160
by auto
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   161
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   162
lemma expand_qsplit:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   163
 "u \<in> A<*>B \<Longrightarrow> R(qsplit(c,u)) \<longleftrightarrow> (\<forall>x\<in>A. \<forall>y\<in>B. u = <x;y> \<longrightarrow> R(c(x,y)))"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   164
apply (simp add: qsplit_def, auto)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   165
done
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   166
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   167
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
   168
subsubsection\<open>qsplit for predicates: result type o\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   169
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   170
lemma qsplitI: "R(a,b) \<Longrightarrow> qsplit(R, <a;b>)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   171
by (simp add: qsplit_def)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   172
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   173
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   174
lemma qsplitE:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   175
    "\<lbrakk>qsplit(R,z);  z \<in> QSigma(A,B);
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   176
        \<And>x y. \<lbrakk>z = <x;y>;  R(x,y)\<rbrakk> \<Longrightarrow> P
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   177
\<rbrakk> \<Longrightarrow> P"
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   178
by (simp add: qsplit_def, auto)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   179
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   180
lemma qsplitD: "qsplit(R,<a;b>) \<Longrightarrow> R(a,b)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   181
by (simp add: qsplit_def)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   182
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   183
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
   184
subsubsection\<open>qconverse\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   185
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   186
lemma qconverseI [intro!]: "<a;b>:r \<Longrightarrow> <b;a>:qconverse(r)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   187
by (simp add: qconverse_def, blast)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   188
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   189
lemma qconverseD [elim!]: "<a;b> \<in> qconverse(r) \<Longrightarrow> <b;a> \<in> r"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   190
by (simp add: qconverse_def, blast)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   191
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   192
lemma qconverseE [elim!]:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   193
    "\<lbrakk>yx \<in> qconverse(r);
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   194
        \<And>x y. \<lbrakk>yx=<y;x>;  <x;y>:r\<rbrakk> \<Longrightarrow> P
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   195
\<rbrakk> \<Longrightarrow> P"
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   196
by (simp add: qconverse_def, blast)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   197
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   198
lemma qconverse_qconverse: "r<=QSigma(A,B) \<Longrightarrow> qconverse(qconverse(r)) = r"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   199
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   200
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   201
lemma qconverse_type: "r \<subseteq> A <*> B \<Longrightarrow> qconverse(r) \<subseteq> B <*> A"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   202
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   203
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   204
lemma qconverse_prod: "qconverse(A <*> B) = B <*> A"
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   205
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   206
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   207
lemma qconverse_empty: "qconverse(0) = 0"
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   208
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   209
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   210
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
   211
subsection\<open>The Quine-inspired notion of disjoint sum\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   212
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   213
lemmas qsum_defs = qsum_def QInl_def QInr_def qcase_def
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   214
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   215
(** Introduction rules for the injections **)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   216
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   217
lemma QInlI [intro!]: "a \<in> A \<Longrightarrow> QInl(a) \<in> A <+> B"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   218
by (simp add: qsum_defs, blast)
1097
01379c46ad2d Changed definitions so that qsplit is now defined in terms of
lcp
parents: 929
diff changeset
   219
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   220
lemma QInrI [intro!]: "b \<in> B \<Longrightarrow> QInr(b) \<in> A <+> B"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   221
by (simp add: qsum_defs, blast)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   222
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   223
(** Elimination rules **)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   224
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   225
lemma qsumE [elim!]:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   226
    "\<lbrakk>u \<in> A <+> B;
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   227
        \<And>x. \<lbrakk>x \<in> A;  u=QInl(x)\<rbrakk> \<Longrightarrow> P;
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   228
        \<And>y. \<lbrakk>y \<in> B;  u=QInr(y)\<rbrakk> \<Longrightarrow> P
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   229
\<rbrakk> \<Longrightarrow> P"
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   230
by (simp add: qsum_defs, blast)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   231
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   232
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   233
(** Injection and freeness equivalences, for rewriting **)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   234
46821
ff6b0c1087f2 Using mathematical notation for <-> and cardinal arithmetic
paulson
parents: 46820
diff changeset
   235
lemma QInl_iff [iff]: "QInl(a)=QInl(b) \<longleftrightarrow> a=b"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   236
by (simp add: qsum_defs )
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   237
46821
ff6b0c1087f2 Using mathematical notation for <-> and cardinal arithmetic
paulson
parents: 46820
diff changeset
   238
lemma QInr_iff [iff]: "QInr(a)=QInr(b) \<longleftrightarrow> a=b"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   239
by (simp add: qsum_defs )
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   240
46821
ff6b0c1087f2 Using mathematical notation for <-> and cardinal arithmetic
paulson
parents: 46820
diff changeset
   241
lemma QInl_QInr_iff [simp]: "QInl(a)=QInr(b) \<longleftrightarrow> False"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   242
by (simp add: qsum_defs )
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   243
46821
ff6b0c1087f2 Using mathematical notation for <-> and cardinal arithmetic
paulson
parents: 46820
diff changeset
   244
lemma QInr_QInl_iff [simp]: "QInr(b)=QInl(a) \<longleftrightarrow> False"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   245
by (simp add: qsum_defs )
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   246
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   247
lemma qsum_empty [simp]: "0<+>0 = 0"
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   248
by (simp add: qsum_defs )
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   249
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   250
(*Injection and freeness rules*)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   251
45602
2a858377c3d2 eliminated obsolete "standard";
wenzelm
parents: 35762
diff changeset
   252
lemmas QInl_inject = QInl_iff [THEN iffD1]
2a858377c3d2 eliminated obsolete "standard";
wenzelm
parents: 35762
diff changeset
   253
lemmas QInr_inject = QInr_iff [THEN iffD1]
13823
d49ffd9f9662 fixed anomalies in the installed classical rules
paulson
parents: 13784
diff changeset
   254
lemmas QInl_neq_QInr = QInl_QInr_iff [THEN iffD1, THEN FalseE, elim!]
d49ffd9f9662 fixed anomalies in the installed classical rules
paulson
parents: 13784
diff changeset
   255
lemmas QInr_neq_QInl = QInr_QInl_iff [THEN iffD1, THEN FalseE, elim!]
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   256
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   257
lemma QInlD: "QInl(a): A<+>B \<Longrightarrow> a \<in> A"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   258
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   259
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   260
lemma QInrD: "QInr(b): A<+>B \<Longrightarrow> b \<in> B"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   261
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   262
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   263
(** <+> is itself injective... who cares?? **)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   264
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   265
lemma qsum_iff:
76214
0c18df79b1c8 more modernisation of syntax
paulson <lp15@cam.ac.uk>
parents: 76213
diff changeset
   266
     "u \<in> A <+> B \<longleftrightarrow> (\<exists>x. x \<in> A \<and> u=QInl(x)) | (\<exists>y. y \<in> B \<and> u=QInr(y))"
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13285
diff changeset
   267
by blast
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   268
76214
0c18df79b1c8 more modernisation of syntax
paulson <lp15@cam.ac.uk>
parents: 76213
diff changeset
   269
lemma qsum_subset_iff: "A <+> B \<subseteq> C <+> D \<longleftrightarrow> A<=C \<and> B<=D"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   270
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   271
76214
0c18df79b1c8 more modernisation of syntax
paulson <lp15@cam.ac.uk>
parents: 76213
diff changeset
   272
lemma qsum_equal_iff: "A <+> B = C <+> D \<longleftrightarrow> A=C \<and> B=D"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   273
apply (simp (no_asm) add: extension qsum_subset_iff)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   274
apply blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   275
done
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   276
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
   277
subsubsection\<open>Eliminator -- qcase\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   278
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   279
lemma qcase_QInl [simp]: "qcase(c, d, QInl(a)) = c(a)"
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   280
by (simp add: qsum_defs )
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   281
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   282
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   283
lemma qcase_QInr [simp]: "qcase(c, d, QInr(b)) = d(b)"
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   284
by (simp add: qsum_defs )
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   286
lemma qcase_type:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   287
    "\<lbrakk>u \<in> A <+> B;
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   288
        \<And>x. x \<in> A \<Longrightarrow> c(x): C(QInl(x));
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   289
        \<And>y. y \<in> B \<Longrightarrow> d(y): C(QInr(y))
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   290
\<rbrakk> \<Longrightarrow> qcase(c,d,u) \<in> C(u)"
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   291
by (simp add: qsum_defs, auto)
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   292
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   293
(** Rules for the Part primitive **)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   294
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   295
lemma Part_QInl: "Part(A <+> B,QInl) = {QInl(x). x \<in> A}"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   296
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   297
46953
2b6e55924af3 replacing ":" by "\<in>"
paulson
parents: 46821
diff changeset
   298
lemma Part_QInr: "Part(A <+> B,QInr) = {QInr(y). y \<in> B}"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   299
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   300
76215
a642599ffdea More syntactic cleanup. LaTeX markup working
paulson <lp15@cam.ac.uk>
parents: 76214
diff changeset
   301
lemma Part_QInr2: "Part(A <+> B, \<lambda>x. QInr(h(x))) = {QInr(y). y \<in> Part(B,h)}"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   302
by blast
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   303
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   304
lemma Part_qsum_equality: "C \<subseteq> A <+> B \<Longrightarrow> Part(C,QInl) \<union> Part(C,QInr) = C"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   305
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   306
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   307
60770
240563fbf41d isabelle update_cartouches;
wenzelm
parents: 58871
diff changeset
   308
subsubsection\<open>Monotonicity\<close>
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   309
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   310
lemma QPair_mono: "\<lbrakk>a<=c;  b<=d\<rbrakk> \<Longrightarrow> <a;b> \<subseteq> <c;d>"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   311
by (simp add: QPair_def sum_mono)
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   312
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   313
lemma QSigma_mono [rule_format]:
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   314
     "\<lbrakk>A<=C;  \<forall>x\<in>A. B(x) \<subseteq> D(x)\<rbrakk> \<Longrightarrow> QSigma(A,B) \<subseteq> QSigma(C,D)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   315
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   316
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   317
lemma QInl_mono: "a<=b \<Longrightarrow> QInl(a) \<subseteq> QInl(b)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   318
by (simp add: QInl_def subset_refl [THEN QPair_mono])
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   319
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   320
lemma QInr_mono: "a<=b \<Longrightarrow> QInr(a) \<subseteq> QInr(b)"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   321
by (simp add: QInr_def subset_refl [THEN QPair_mono])
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   322
76213
e44d86131648 Removal of obsolete ASCII syntax
paulson <lp15@cam.ac.uk>
parents: 69587
diff changeset
   323
lemma qsum_mono: "\<lbrakk>A<=C;  B<=D\<rbrakk> \<Longrightarrow> A <+> B \<subseteq> C <+> D"
13285
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   324
by blast
28d1823ce0f2 conversion of QPair to Isar
paulson
parents: 13259
diff changeset
   325
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   326
end