src/HOLCF/ex/Focus_ex.thy
author wenzelm
Sun, 21 Oct 2007 16:27:42 +0200
changeset 25135 4f8176c940cf
parent 21404 eb85850d3eb7
child 27185 0407630909ef
permissions -rw-r--r--
modernized specifications ('definition', 'axiomatization');
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
     1
(* $Id$ *)
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
     2
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
     3
(* Specification of the following loop back device
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
     4
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
     5
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
     6
          g
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
     7
           --------------------
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
     8
          |      -------       |
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
     9
       x  |     |       |      |  y
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    10
    ------|---->|       |------| ----->
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    11
          |  z  |   f   | z    |
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    12
          |  -->|       |---   |
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    13
          | |   |       |   |  |
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    14
          | |    -------    |  |
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    15
          | |               |  |
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    16
          |  <--------------   |
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    17
          |                    |
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    18
           --------------------
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    19
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    20
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    21
First step: Notation in Agent Network Description Language (ANDL)
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    22
-----------------------------------------------------------------
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    23
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    24
agent f
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    25
        input  channel i1:'b i2: ('b,'c) tc
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    26
        output channel o1:'c o2: ('b,'c) tc
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    27
is
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    28
        Rf(i1,i2,o1,o2)  (left open in the example)
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    29
end f
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    30
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    31
agent g
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    32
        input  channel x:'b
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    33
        output channel y:'c
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    34
is network
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    35
        <y,z> = f$<x,z>
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    36
end network
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    37
end g
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    38
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    39
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    40
Remark: the type of the feedback depends at most on the types of the input and
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    41
        output of g. (No type miracles inside g)
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    42
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    43
Second step: Translation of ANDL specification to HOLCF Specification
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    44
---------------------------------------------------------------------
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    45
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    46
Specification of agent f ist translated to predicate is_f
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    47
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    48
is_f :: ('b stream * ('b,'c) tc stream ->
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    49
                'c stream * ('b,'c) tc stream) => bool
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    50
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    51
is_f f  = !i1 i2 o1 o2.
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    52
        f$<i1,i2> = <o1,o2> --> Rf(i1,i2,o1,o2)
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    53
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    54
Specification of agent g is translated to predicate is_g which uses
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    55
predicate is_net_g
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    56
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    57
is_net_g :: ('b stream * ('b,'c) tc stream -> 'c stream * ('b,'c) tc stream) =>
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    58
            'b stream => 'c stream => bool
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    59
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    60
is_net_g f x y =
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    61
        ? z. <y,z> = f$<x,z> &
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    62
        !oy hz. <oy,hz> = f$<x,hz> --> z << hz
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    63
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    64
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    65
is_g :: ('b stream -> 'c stream) => bool
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    66
10835
nipkow
parents: 3842
diff changeset
    67
is_g g  = ? f. is_f f  & (!x y. g$x = y --> is_net_g f x y
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    68
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    69
Third step: (show conservativity)
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    70
-----------
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    71
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    72
Suppose we have a model for the theory TH1 which contains the axiom
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    73
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    74
        ? f. is_f f
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    75
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    76
In this case there is also a model for the theory TH2 that enriches TH1 by
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    77
axiom
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    78
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    79
        ? g. is_g g
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    80
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    81
The result is proved by showing that there is a definitional extension
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    82
that extends TH1 by a definition of g.
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    83
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    84
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    85
We define:
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    86
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    87
def_g g  =
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    88
         (? f. is_f f  &
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    89
              g = (LAM x. cfst$(f$<x,fix$(LAM k.csnd$(f$<x,k>))>)) )
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    90
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    91
Now we prove:
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    92
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    93
        (? f. is_f f ) --> (? g. is_g g)
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    94
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    95
using the theorems
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    96
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    97
loopback_eq)    def_g = is_g                    (real work)
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
    98
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
    99
L1)             (? f. is_f f ) --> (? g. def_g g)  (trivial)
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   100
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   101
*)
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   102
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
   103
theory Focus_ex
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
   104
imports Stream
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
   105
begin
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   106
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
   107
typedecl ('a, 'b) tc
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
   108
arities tc:: (pcpo, pcpo) pcpo
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   109
25135
4f8176c940cf modernized specifications ('definition', 'axiomatization');
wenzelm
parents: 21404
diff changeset
   110
axiomatization
19763
wenzelm
parents: 19742
diff changeset
   111
  Rf :: "('b stream * ('b,'c) tc stream * 'c stream * ('b,'c) tc stream) => bool"
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   112
19763
wenzelm
parents: 19742
diff changeset
   113
definition
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19763
diff changeset
   114
  is_f :: "('b stream * ('b,'c) tc stream -> 'c stream * ('b,'c) tc stream) => bool" where
19763
wenzelm
parents: 19742
diff changeset
   115
  "is_f f = (!i1 i2 o1 o2. f$<i1,i2> = <o1,o2> --> Rf(i1,i2,o1,o2))"
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   116
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19763
diff changeset
   117
definition
19763
wenzelm
parents: 19742
diff changeset
   118
  is_net_g :: "('b stream *('b,'c) tc stream -> 'c stream * ('b,'c) tc stream) =>
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19763
diff changeset
   119
    'b stream => 'c stream => bool" where
19763
wenzelm
parents: 19742
diff changeset
   120
  "is_net_g f x y == (? z.
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
   121
                        <y,z> = f$<x,z> &
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
   122
                        (!oy hz. <oy,hz> = f$<x,hz> --> z << hz))"
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   123
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19763
diff changeset
   124
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19763
diff changeset
   125
  is_g :: "('b stream -> 'c stream) => bool" where
19763
wenzelm
parents: 19742
diff changeset
   126
  "is_g g  == (? f. is_f f  & (!x y. g$x = y --> is_net_g f x y))"
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   127
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19763
diff changeset
   128
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19763
diff changeset
   129
  def_g :: "('b stream -> 'c stream) => bool" where
19763
wenzelm
parents: 19742
diff changeset
   130
  "def_g g == (? f. is_f f  & g = (LAM x. cfst$(f$<x,fix$(LAM  k. csnd$(f$<x,k>))>)))"
17291
94f6113fe9ed converted to Isar theory format;
wenzelm
parents: 10835
diff changeset
   131
19742
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   132
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   133
(* first some logical trading *)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   134
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   135
lemma lemma1:
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   136
"is_g(g) =
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   137
  (? f. is_f(f) &  (!x.(? z. <g$x,z> = f$<x,z> &
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   138
                   (! w y. <y,w> = f$<x,w>  --> z << w))))"
19763
wenzelm
parents: 19742
diff changeset
   139
apply (simp add: is_g_def is_net_g_def)
19742
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   140
apply fast
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   141
done
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   142
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   143
lemma lemma2:
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   144
"(? f. is_f(f) &  (!x. (? z. <g$x,z> = f$<x,z> &
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   145
                  (!w y. <y,w> = f$<x,w>  --> z << w))))
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   146
  =
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   147
  (? f. is_f(f) &  (!x. ? z.
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   148
        g$x = cfst$(f$<x,z>) &
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   149
          z = csnd$(f$<x,z>) &
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   150
        (! w y.  <y,w> = f$<x,w> --> z << w)))"
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   151
apply (rule iffI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   152
apply (erule exE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   153
apply (rule_tac x = "f" in exI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   154
apply (erule conjE)+
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   155
apply (erule conjI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   156
apply (intro strip)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   157
apply (erule allE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   158
apply (erule exE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   159
apply (rule_tac x = "z" in exI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   160
apply (erule conjE)+
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   161
apply (rule conjI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   162
apply (rule_tac [2] conjI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   163
prefer 3 apply (assumption)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   164
apply (drule sym)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   165
apply (tactic "asm_simp_tac HOLCF_ss 1")
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   166
apply (drule sym)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   167
apply (tactic "asm_simp_tac HOLCF_ss 1")
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   168
apply (erule exE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   169
apply (rule_tac x = "f" in exI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   170
apply (erule conjE)+
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   171
apply (erule conjI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   172
apply (intro strip)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   173
apply (erule allE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   174
apply (erule exE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   175
apply (rule_tac x = "z" in exI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   176
apply (erule conjE)+
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   177
apply (rule conjI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   178
prefer 2 apply (assumption)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   179
apply (rule trans)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   180
apply (rule_tac [2] surjective_pairing_Cprod2)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   181
apply (erule subst)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   182
apply (erule subst)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   183
apply (rule refl)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   184
done
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   185
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   186
lemma lemma3: "def_g(g) --> is_g(g)"
19763
wenzelm
parents: 19742
diff changeset
   187
apply (tactic {* simp_tac (HOL_ss addsimps [thm "def_g_def", thm "lemma1", thm "lemma2"]) 1 *})
19742
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   188
apply (rule impI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   189
apply (erule exE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   190
apply (rule_tac x = "f" in exI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   191
apply (erule conjE)+
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   192
apply (erule conjI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   193
apply (intro strip)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   194
apply (rule_tac x = "fix$ (LAM k. csnd$ (f$<x,k>))" in exI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   195
apply (rule conjI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   196
 apply (tactic "asm_simp_tac HOLCF_ss 1")
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   197
 apply (rule trans)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   198
  apply (rule_tac [2] surjective_pairing_Cprod2)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   199
 apply (rule cfun_arg_cong)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   200
 apply (rule trans)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   201
  apply (rule fix_eq)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   202
 apply (simp (no_asm))
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   203
apply (intro strip)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   204
apply (rule fix_least)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   205
apply (simp (no_asm))
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   206
apply (erule exE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   207
apply (drule sym)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   208
back
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   209
apply simp
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   210
done
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   211
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   212
lemma lemma4: "is_g(g) --> def_g(g)"
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   213
apply (tactic {* simp_tac (HOL_ss delsimps (thms "ex_simps" @ thms "all_simps")
19763
wenzelm
parents: 19742
diff changeset
   214
  addsimps [thm "lemma1", thm "lemma2", thm "def_g_def"]) 1 *})
19742
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   215
apply (rule impI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   216
apply (erule exE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   217
apply (rule_tac x = "f" in exI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   218
apply (erule conjE)+
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   219
apply (erule conjI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   220
apply (rule ext_cfun)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   221
apply (erule_tac x = "x" in allE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   222
apply (erule exE)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   223
apply (erule conjE)+
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   224
apply (subgoal_tac "fix$ (LAM k. csnd$ (f$<x, k>)) = z")
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   225
 apply simp
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   226
apply (subgoal_tac "! w y. f$<x, w> = <y, w> --> z << w")
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   227
apply (rule sym)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   228
apply (rule fix_eqI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   229
apply simp
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   230
apply (rule allI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   231
apply (tactic "simp_tac HOLCF_ss 1")
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   232
apply (intro strip)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   233
apply (subgoal_tac "f$<x, za> = <cfst$ (f$<x,za>) ,za>")
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   234
apply fast
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   235
apply (rule trans)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   236
apply (rule surjective_pairing_Cprod2 [symmetric])
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   237
apply (erule cfun_arg_cong)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   238
apply (intro strip)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   239
apply (erule allE)+
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   240
apply (erule mp)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   241
apply (erule sym)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   242
done
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   243
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   244
(* now we assemble the result *)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   245
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   246
lemma loopback_eq: "def_g = is_g"
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   247
apply (rule ext)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   248
apply (rule iffI)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   249
apply (erule lemma3 [THEN mp])
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   250
apply (erule lemma4 [THEN mp])
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   251
done
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   252
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   253
lemma L2:
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   254
"(? f.
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   255
  is_f(f::'b stream * ('b,'c) tc stream -> 'c stream * ('b,'c) tc stream))
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   256
  -->
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   257
  (? g. def_g(g::'b stream -> 'c stream ))"
19763
wenzelm
parents: 19742
diff changeset
   258
apply (simp add: def_g_def)
19742
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   259
done
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   260
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   261
theorem conservative_loopback:
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   262
"(? f.
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   263
  is_f(f::'b stream * ('b,'c) tc stream -> 'c stream * ('b,'c) tc stream))
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   264
  -->
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   265
  (? g. is_g(g::'b stream -> 'c stream ))"
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   266
apply (rule loopback_eq [THEN subst])
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   267
apply (rule L2)
86f21beabafc removed legacy ML scripts;
wenzelm
parents: 17291
diff changeset
   268
done
2570
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   269
24d7e8fb8261 added Classlib.* and Witness.*,
oheimb
parents:
diff changeset
   270
end