src/HOLCF/Ssum3.ML
author wenzelm
Fri, 06 Oct 2000 17:35:58 +0200
changeset 10168 50be659d4222
parent 9248 e1dee89de037
child 10198 2b255b772585
permissions -rw-r--r--
final tuning;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
     1
(*  Title:      HOLCF/Ssum3.ML
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
     2
    ID:         $Id$
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 1277
diff changeset
     3
    Author:     Franz Regensburger
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
     4
    Copyright   1993 Technische Universitaet Muenchen
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
     5
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
     6
Class instance of  ++ for class pcpo
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
     7
*)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
     8
2640
ee4dfce170a0 Changes of HOLCF from Oscar Slotosch:
slotosch
parents: 2566
diff changeset
     9
(* for compatibility with old HOLCF-Version *)
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    10
Goal "UU = Isinl UU";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    11
by (simp_tac (HOL_ss addsimps [UU_def,UU_ssum_def]) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    12
qed "inst_ssum_pcpo";
2640
ee4dfce170a0 Changes of HOLCF from Oscar Slotosch:
slotosch
parents: 2566
diff changeset
    13
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    14
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    15
(* continuity for Isinl and Isinr                                           *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    16
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    17
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    18
Goal "contlub(Isinl)";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    19
by (rtac contlubI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    20
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    21
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    22
by (rtac (thelub_ssum1a RS sym) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    23
by (rtac allI 3);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    24
by (rtac exI 3);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    25
by (rtac refl 3);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    26
by (etac (monofun_Isinl RS ch2ch_monofun) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    27
by (case_tac "lub(range(Y))=UU" 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    28
by (res_inst_tac [("s","UU"),("t","lub(range(Y))")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    29
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    30
by (res_inst_tac [("f","Isinl")] arg_cong  1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    31
by (rtac (chain_UU_I_inverse RS sym) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    32
by (rtac allI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    33
by (res_inst_tac [("s","UU"),("t","Y(i)")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    34
by (etac (chain_UU_I RS spec ) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    35
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    36
by (rtac Iwhen1 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    37
by (res_inst_tac [("f","Isinl")] arg_cong  1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    38
by (rtac lub_equal 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    39
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    40
by (rtac (monofun_Iwhen3 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    41
by (etac (monofun_Isinl RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    42
by (rtac allI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    43
by (case_tac "Y(k)=UU" 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    44
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    45
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    46
qed "contlub_Isinl";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    47
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    48
Goal "contlub(Isinr)";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    49
by (rtac contlubI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    50
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    51
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    52
by (rtac (thelub_ssum1b RS sym) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    53
by (rtac allI 3);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    54
by (rtac exI 3);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    55
by (rtac refl 3);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    56
by (etac (monofun_Isinr RS ch2ch_monofun) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    57
by (case_tac "lub(range(Y))=UU" 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    58
by (res_inst_tac [("s","UU"),("t","lub(range(Y))")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    59
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    60
by ((rtac arg_cong 1) THEN (rtac (chain_UU_I_inverse RS sym) 1));
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    61
by (rtac allI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    62
by (res_inst_tac [("s","UU"),("t","Y(i)")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    63
by (etac (chain_UU_I RS spec ) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    64
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    65
by (rtac (strict_IsinlIsinr RS subst) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    66
by (rtac Iwhen1 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    67
by ((rtac arg_cong 1) THEN (rtac lub_equal 1));
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    68
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    69
by (rtac (monofun_Iwhen3 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    70
by (etac (monofun_Isinr RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    71
by (rtac allI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    72
by (case_tac "Y(k)=UU" 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    73
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    74
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    75
qed "contlub_Isinr";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    76
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    77
Goal "cont(Isinl)";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    78
by (rtac monocontlub2cont 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    79
by (rtac monofun_Isinl 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    80
by (rtac contlub_Isinl 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    81
qed "cont_Isinl";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    82
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    83
Goal "cont(Isinr)";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    84
by (rtac monocontlub2cont 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    85
by (rtac monofun_Isinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    86
by (rtac contlub_Isinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    87
qed "cont_Isinr";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    88
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
    89
AddIffs [cont_Isinl, cont_Isinr];
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
    90
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    91
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    92
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    93
(* continuity for Iwhen in the firts two arguments                          *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    94
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
    95
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    96
Goal "contlub(Iwhen)";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    97
by (rtac contlubI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    98
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
    99
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   100
by (rtac (thelub_fun RS sym) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   101
by (etac (monofun_Iwhen1 RS ch2ch_monofun) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   102
by (rtac (expand_fun_eq RS iffD2) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   103
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   104
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   105
by (rtac (thelub_fun RS sym) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   106
by (rtac ch2ch_fun 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   107
by (etac (monofun_Iwhen1 RS ch2ch_monofun) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   108
by (rtac (expand_fun_eq RS iffD2) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   109
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   110
by (res_inst_tac [("p","xa")] IssumE 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   111
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   112
by (rtac (lub_const RS thelubI RS sym) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   113
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   114
by (etac contlub_cfun_fun 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   115
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   116
by (rtac (lub_const RS thelubI RS sym) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   117
qed "contlub_Iwhen1";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   118
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   119
Goal "contlub(Iwhen(f))";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   120
by (rtac contlubI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   121
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   122
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   123
by (rtac (thelub_fun RS sym) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   124
by (etac (monofun_Iwhen2 RS ch2ch_monofun) 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   125
by (rtac (expand_fun_eq RS iffD2) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   126
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   127
by (res_inst_tac [("p","x")] IssumE 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   128
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   129
by (rtac (lub_const RS thelubI RS sym) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   130
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   131
by (rtac (lub_const RS thelubI RS sym) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   132
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   133
by (etac contlub_cfun_fun 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   134
qed "contlub_Iwhen2";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   135
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   136
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   137
(* continuity for Iwhen in its third argument                               *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   138
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   139
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   140
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   141
(* first 5 ugly lemmas                                                      *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   142
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   143
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   144
Goal "[| chain(Y); lub(range(Y)) = Isinl(x)|] ==> !i.? x. Y(i)=Isinl(x)";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   145
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   146
by (res_inst_tac [("p","Y(i)")] IssumE 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   147
by (etac exI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   148
by (etac exI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   149
by (res_inst_tac [("P","y=UU")] notE 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   150
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   151
by (rtac (less_ssum3d RS iffD1) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   152
by (etac subst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   153
by (etac subst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   154
by (etac is_ub_thelub 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   155
qed "ssum_lemma9";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   156
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   157
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   158
Goal "[| chain(Y); lub(range(Y)) = Isinr(x)|] ==> !i.? x. Y(i)=Isinr(x)";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   159
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   160
by (res_inst_tac [("p","Y(i)")] IssumE 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   161
by (rtac exI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   162
by (etac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   163
by (rtac strict_IsinlIsinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   164
by (etac exI 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   165
by (res_inst_tac [("P","xa=UU")] notE 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   166
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   167
by (rtac (less_ssum3c RS iffD1) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   168
by (etac subst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   169
by (etac subst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   170
by (etac is_ub_thelub 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   171
qed "ssum_lemma10";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   172
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   173
Goal "[| chain(Y); lub(range(Y)) = Isinl(UU) |] ==>\
8161
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   174
\   Iwhen f g (lub(range Y)) = lub(range(%i. Iwhen f g (Y i)))";
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   175
by (asm_simp_tac Ssum0_ss 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   176
by (rtac (chain_UU_I_inverse RS sym) 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   177
by (rtac allI 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   178
by (res_inst_tac [("s","Isinl(UU)"),("t","Y(i)")] subst 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   179
by (rtac (inst_ssum_pcpo RS subst) 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   180
by (rtac (chain_UU_I RS spec RS sym) 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   181
by (atac 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   182
by (etac (inst_ssum_pcpo RS ssubst) 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   183
by (asm_simp_tac Ssum0_ss 1);
bde1391fd0a5 added range_composition (also to simpset)
oheimb
parents: 5439
diff changeset
   184
qed "ssum_lemma11";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   185
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   186
Goal "[| chain(Y); lub(range(Y)) = Isinl(x); x ~= UU |] ==>\
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   187
\   Iwhen f g (lub(range Y)) = lub(range(%i. Iwhen f g (Y i)))";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   188
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   189
by (res_inst_tac [("t","x")] subst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   190
by (rtac inject_Isinl 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   191
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   192
by (atac 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   193
by (rtac (thelub_ssum1a RS sym) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   194
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   195
by (etac ssum_lemma9 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   196
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   197
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   198
by (rtac contlub_cfun_arg 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   199
by (rtac (monofun_Iwhen3 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   200
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   201
by (rtac lub_equal2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   202
by (rtac (chain_mono2 RS exE) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   203
by (atac 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   204
by (rtac chain_UU_I_inverse2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   205
by (stac inst_ssum_pcpo 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   206
by (etac swap 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   207
by (rtac inject_Isinl 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   208
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   209
by (etac sym 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   210
by (etac notnotD 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   211
by (rtac exI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   212
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   213
by (rtac (ssum_lemma9 RS spec RS exE) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   214
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   215
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   216
by (res_inst_tac [("t","Y(i)")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   217
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   218
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   219
by (rtac cfun_arg_cong 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   220
by (rtac Iwhen2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   221
by (res_inst_tac [("Pa","Y(i)=UU")] swap 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   222
by (fast_tac HOL_cs 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   223
by (stac inst_ssum_pcpo 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   224
by (res_inst_tac [("t","Y(i)")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   225
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   226
by (fast_tac HOL_cs 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   227
by (stac Iwhen2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   228
by (res_inst_tac [("Pa","Y(i)=UU")] swap 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   229
by (fast_tac HOL_cs 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   230
by (stac inst_ssum_pcpo 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   231
by (res_inst_tac [("t","Y(i)")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   232
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   233
by (fast_tac HOL_cs 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   234
by (simp_tac (simpset_of Cfun3.thy) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   235
by (rtac (monofun_Rep_CFun2 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   236
by (etac (monofun_Iwhen3 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   237
by (etac (monofun_Iwhen3 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   238
qed "ssum_lemma12";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   239
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   240
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   241
Goal "[| chain(Y); lub(range(Y)) = Isinr(x); x ~= UU |] ==>\
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   242
\   Iwhen f g (lub(range Y)) = lub(range(%i. Iwhen f g (Y i)))";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   243
by (asm_simp_tac Ssum0_ss 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   244
by (res_inst_tac [("t","x")] subst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   245
by (rtac inject_Isinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   246
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   247
by (atac 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   248
by (rtac (thelub_ssum1b RS sym) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   249
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   250
by (etac ssum_lemma10 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   251
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   252
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   253
by (rtac contlub_cfun_arg 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   254
by (rtac (monofun_Iwhen3 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   255
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   256
by (rtac lub_equal2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   257
by (rtac (chain_mono2 RS exE) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   258
by (atac 2);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   259
by (rtac chain_UU_I_inverse2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   260
by (stac inst_ssum_pcpo 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   261
by (etac swap 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   262
by (rtac inject_Isinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   263
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   264
by (etac sym 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   265
by (rtac (strict_IsinlIsinr RS subst) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   266
by (etac notnotD 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   267
by (rtac exI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   268
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   269
by (rtac (ssum_lemma10 RS spec RS exE) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   270
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   271
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   272
by (res_inst_tac [("t","Y(i)")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   273
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   274
by (rtac trans 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   275
by (rtac cfun_arg_cong 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   276
by (rtac Iwhen3 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   277
by (res_inst_tac [("Pa","Y(i)=UU")] swap 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   278
by (fast_tac HOL_cs 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   279
by (dtac notnotD 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   280
by (stac inst_ssum_pcpo 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   281
by (stac strict_IsinlIsinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   282
by (res_inst_tac [("t","Y(i)")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   283
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   284
by (fast_tac HOL_cs 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   285
by (stac Iwhen3 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   286
by (res_inst_tac [("Pa","Y(i)=UU")] swap 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   287
by (fast_tac HOL_cs 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   288
by (dtac notnotD 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   289
by (stac inst_ssum_pcpo 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   290
by (stac strict_IsinlIsinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   291
by (res_inst_tac [("t","Y(i)")] ssubst 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   292
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   293
by (fast_tac HOL_cs 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   294
by (simp_tac (simpset_of Cfun3.thy) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   295
by (rtac (monofun_Rep_CFun2 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   296
by (etac (monofun_Iwhen3 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   297
by (etac (monofun_Iwhen3 RS ch2ch_monofun) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   298
qed "ssum_lemma13";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   299
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   300
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   301
Goal "contlub(Iwhen(f)(g))";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   302
by (rtac contlubI 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   303
by (strip_tac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   304
by (res_inst_tac [("p","lub(range(Y))")] IssumE 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   305
by (etac ssum_lemma11 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   306
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   307
by (etac ssum_lemma12 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   308
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   309
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   310
by (etac ssum_lemma13 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   311
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   312
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   313
qed "contlub_Iwhen3";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   314
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   315
Goal "cont(Iwhen)";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   316
by (rtac monocontlub2cont 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   317
by (rtac monofun_Iwhen1 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   318
by (rtac contlub_Iwhen1 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   319
qed "cont_Iwhen1";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   320
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   321
Goal "cont(Iwhen(f))";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   322
by (rtac monocontlub2cont 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   323
by (rtac monofun_Iwhen2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   324
by (rtac contlub_Iwhen2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   325
qed "cont_Iwhen2";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   326
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   327
Goal "cont(Iwhen(f)(g))";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   328
by (rtac monocontlub2cont 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   329
by (rtac monofun_Iwhen3 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   330
by (rtac contlub_Iwhen3 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   331
qed "cont_Iwhen3";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   332
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   333
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   334
(* continuous versions of lemmas for 'a ++ 'b                               *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   335
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   336
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   337
Goalw [sinl_def] "sinl`UU =UU";
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   338
by (simp_tac (Ssum0_ss addsimps [cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   339
by (rtac (inst_ssum_pcpo RS sym) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   340
qed "strict_sinl";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   341
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   342
Goalw [sinr_def] "sinr`UU=UU";
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   343
by (simp_tac (Ssum0_ss addsimps [cont_Isinr]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   344
by (rtac (inst_ssum_pcpo RS sym) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   345
qed "strict_sinr";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   346
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   347
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   348
        "sinl`a=sinr`b ==> a=UU & b=UU";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   349
by (rtac noteq_IsinlIsinr 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   350
by (etac box_equals 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   351
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   352
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   353
qed "noteq_sinlsinr";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   354
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   355
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   356
        "sinl`a1=sinl`a2==> a1=a2";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   357
by (rtac inject_Isinl 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   358
by (etac box_equals 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   359
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   360
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   361
qed "inject_sinl";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   362
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   363
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   364
        "sinr`a1=sinr`a2==> a1=a2";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   365
by (rtac inject_Isinr 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   366
by (etac box_equals 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   367
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   368
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   369
qed "inject_sinr";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   370
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   371
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   372
Goal "x~=UU ==> sinl`x ~= UU";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   373
by (etac swap 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   374
by (rtac inject_sinl 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   375
by (stac strict_sinl 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   376
by (etac notnotD 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   377
qed "defined_sinl";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   378
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   379
Goal "x~=UU ==> sinr`x ~= UU";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   380
by (etac swap 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   381
by (rtac inject_sinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   382
by (stac strict_sinr 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   383
by (etac notnotD 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   384
qed "defined_sinr";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   385
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   386
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   387
        "z=UU | (? a. z=sinl`a & a~=UU) | (? b. z=sinr`b & b~=UU)";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   388
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   389
by (stac inst_ssum_pcpo 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   390
by (rtac Exh_Ssum 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   391
qed "Exh_Ssum1";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   392
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   393
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   394
val [major,prem2,prem3] = Goalw [sinl_def,sinr_def] 
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 1277
diff changeset
   395
        "[|p=UU ==> Q ;\
6bcb44e4d6e5 expanded tabs
clasohm
parents: 1277
diff changeset
   396
\       !!x.[|p=sinl`x; x~=UU |] ==> Q;\
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   397
\       !!y.[|p=sinr`y; y~=UU |] ==> Q|] ==> Q";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   398
by (rtac (major RS IssumE) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   399
by (stac inst_ssum_pcpo 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   400
by (atac 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   401
by (rtac prem2 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   402
by (atac 2);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   403
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   404
by (rtac prem3 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   405
by (atac 2);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   406
by (Asm_simp_tac 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   407
qed "ssumE";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   408
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   409
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   410
val [preml,premr] = Goalw [sinl_def,sinr_def] 
1168
74be52691d62 The curried version of HOLCF is now just called HOLCF. The old
regensbu
parents: 892
diff changeset
   411
      "[|!!x.[|p=sinl`x|] ==> Q;\
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   412
\        !!y.[|p=sinr`y|] ==> Q|] ==> Q";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   413
by (rtac IssumE2 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   414
by (rtac preml 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   415
by (rtac premr 2);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   416
by Auto_tac;  
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   417
qed "ssumE2";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   418
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   419
val tac = (REPEAT (resolve_tac (cont_lemmas1 @ [cont_Iwhen1,cont_Iwhen2,
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   420
                cont_Iwhen3,cont2cont_CF1L]) 1)); 
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   421
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   422
Goalw [sscase_def,sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   423
        "sscase`f`g`UU = UU";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   424
by (stac inst_ssum_pcpo 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   425
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   426
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   427
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   428
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   429
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   430
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   431
by (simp_tac Ssum0_ss  1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   432
qed "sscase1";
2566
cbf02fc74332 changed handling of cont_lemmas and adm_lemmas
oheimb
parents: 2033
diff changeset
   433
cbf02fc74332 changed handling of cont_lemmas and adm_lemmas
oheimb
parents: 2033
diff changeset
   434
cbf02fc74332 changed handling of cont_lemmas and adm_lemmas
oheimb
parents: 2033
diff changeset
   435
val tac = (REPEAT (resolve_tac (cont_lemmas1 @ [cont_Iwhen1,cont_Iwhen2,
cbf02fc74332 changed handling of cont_lemmas and adm_lemmas
oheimb
parents: 2033
diff changeset
   436
                cont_Iwhen3,cont_Isinl,cont_Isinr,cont2cont_CF1L]) 1));
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   437
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   438
Goalw [sscase_def,sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   439
        "x~=UU==> sscase`f`g`(sinl`x) = f`x";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   440
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   441
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   442
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   443
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   444
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   445
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   446
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   447
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   448
by (asm_simp_tac Ssum0_ss  1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   449
qed "sscase2";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   450
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   451
Goalw [sscase_def,sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   452
        "x~=UU==> sscase`f`g`(sinr`x) = g`x";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   453
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   454
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   455
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   456
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   457
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   458
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   459
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   460
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   461
by (asm_simp_tac Ssum0_ss  1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   462
qed "sscase3";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   463
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   464
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   465
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   466
        "(sinl`x << sinl`y) = (x << y)";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   467
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   468
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   469
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   470
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   471
by (rtac less_ssum3a 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   472
qed "less_ssum4a";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   473
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   474
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   475
        "(sinr`x << sinr`y) = (x << y)";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   476
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   477
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   478
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   479
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   480
by (rtac less_ssum3b 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   481
qed "less_ssum4b";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   482
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   483
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   484
        "(sinl`x << sinr`y) = (x = UU)";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   485
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   486
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   487
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   488
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   489
by (rtac less_ssum3c 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   490
qed "less_ssum4c";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   491
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   492
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   493
        "(sinr`x << sinl`y) = (x = UU)";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   494
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   495
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   496
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   497
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   498
by (rtac less_ssum3d 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   499
qed "less_ssum4d";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   500
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   501
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   502
        "chain(Y) ==> (!i.? x.(Y i)=sinl`x)|(!i.? y.(Y i)=sinr`y)";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   503
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   504
by (etac ssum_lemma4 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   505
qed "ssum_chainE";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   506
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   507
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   508
Goalw [sinl_def,sinr_def,sscase_def] 
4721
c8a8482a8124 renamed is_chain to chain, is_tord to tord, replaced chain_finite by chfin
oheimb
parents: 4098
diff changeset
   509
"[| chain(Y); !i.? x. Y(i) = sinl`x |] ==>\ 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   510
\   lub(range(Y)) = sinl`(lub(range(%i. sscase`(LAM x. x)`(LAM y. UU)`(Y i))))";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   511
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   512
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   513
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   514
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   515
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   516
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   517
by (stac (beta_cfun RS ext) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   518
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   519
by (rtac thelub_ssum1a 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   520
by (atac 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   521
by (rtac allI 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   522
by (etac allE 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   523
by (etac exE 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   524
by (rtac exI 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   525
by (etac box_equals 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   526
by (rtac refl 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   527
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinl]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   528
qed "thelub_ssum2a";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   529
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   530
Goalw [sinl_def,sinr_def,sscase_def] 
4721
c8a8482a8124 renamed is_chain to chain, is_tord to tord, replaced chain_finite by chfin
oheimb
parents: 4098
diff changeset
   531
"[| chain(Y); !i.? x. Y(i) = sinr`x |] ==>\ 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   532
\   lub(range(Y)) = sinr`(lub(range(%i. sscase`(LAM y. UU)`(LAM x. x)`(Y i))))";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   533
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   534
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   535
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   536
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   537
by (stac beta_cfun 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   538
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   539
by (stac (beta_cfun RS ext) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   540
by tac;
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   541
by (rtac thelub_ssum1b 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   542
by (atac 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   543
by (rtac allI 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   544
by (etac allE 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   545
by (etac exE 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   546
by (rtac exI 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   547
by (etac box_equals 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   548
by (rtac refl 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   549
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl,cont_Iwhen1,cont_Iwhen2, cont_Iwhen3]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   550
qed "thelub_ssum2b";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   551
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   552
Goalw [sinl_def,sinr_def] 
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   553
        "[| chain(Y); lub(range(Y)) = sinl`x|] ==> !i.? x. Y(i)=sinl`x";
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   554
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl,cont_Iwhen1,cont_Iwhen2, cont_Iwhen3]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   555
by (etac ssum_lemma9 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   556
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl,cont_Iwhen1,cont_Iwhen2, cont_Iwhen3]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   557
qed "thelub_ssum2a_rev";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   558
9248
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   559
Goalw [sinl_def,sinr_def] 
e1dee89de037 massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents: 9245
diff changeset
   560
     "[| chain(Y); lub(range(Y)) = sinr`x|] ==> !i.? x. Y(i)=sinr`x";
9245
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   561
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl,cont_Iwhen1,cont_Iwhen2, cont_Iwhen3]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   562
by (etac ssum_lemma10 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   563
by (asm_simp_tac (Ssum0_ss addsimps [cont_Isinr,cont_Isinl,cont_Iwhen1,cont_Iwhen2, cont_Iwhen3]) 1);
428385c4bc50 removed most batch-style proofs
paulson
parents: 9169
diff changeset
   564
qed "thelub_ssum2b_rev";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   565
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   566
Goal "chain(Y) ==>\ 
5439
2e0c18eedfd0 renamed sswhen to sscase
oheimb
parents: 5291
diff changeset
   567
\   lub(range(Y)) = sinl`(lub(range(%i. sscase`(LAM x. x)`(LAM y. UU)`(Y i))))\
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   568
\ | lub(range(Y)) = sinr`(lub(range(%i. sscase`(LAM y. UU)`(LAM x. x)`(Y i))))";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   569
by (rtac (ssum_chainE RS disjE) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   570
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   571
by (rtac disjI1 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   572
by (etac thelub_ssum2a 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   573
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   574
by (rtac disjI2 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   575
by (etac thelub_ssum2b 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   576
by (atac 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   577
qed "thelub_ssum3";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   578
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   579
9169
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   580
Goal "sscase`sinl`sinr`z=z";
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   581
by (res_inst_tac [("p","z")] ssumE 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   582
by (asm_simp_tac ((simpset_of Cfun3.thy) addsimps [sscase1,sscase2,sscase3]) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   583
by (asm_simp_tac ((simpset_of Cfun3.thy) addsimps [sscase1,sscase2,sscase3]) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   584
by (asm_simp_tac ((simpset_of Cfun3.thy) addsimps [sscase1,sscase2,sscase3]) 1);
85a47aa21f74 tidying and unbatchifying
paulson
parents: 8161
diff changeset
   585
qed "sscase4";
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   586
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   587
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   588
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   589
(* install simplifier for Ssum                                              *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   590
(* ------------------------------------------------------------------------ *)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
   591
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents: 1267
diff changeset
   592
val Ssum_rews = [strict_sinl,strict_sinr,defined_sinl,defined_sinr,
5439
2e0c18eedfd0 renamed sswhen to sscase
oheimb
parents: 5291
diff changeset
   593
                sscase1,sscase2,sscase3];
1274
ea0668a1c0ba added 8bit pragmas
regensbu
parents: 1267
diff changeset
   594
ea0668a1c0ba added 8bit pragmas
regensbu
parents: 1267
diff changeset
   595
Addsimps [strict_sinl,strict_sinr,defined_sinl,defined_sinr,
5439
2e0c18eedfd0 renamed sswhen to sscase
oheimb
parents: 5291
diff changeset
   596
                sscase1,sscase2,sscase3];