src/ZF/WF.thy
author skalberg
Thu, 28 Aug 2003 01:56:40 +0200
changeset 14171 0cab06e3bbd0
parent 13784 b9f6154427a4
child 16417 9bc16273c2d4
permissions -rw-r--r--
Extended the notion of letter and digit, such that now one may use greek, gothic, euler, or calligraphic letters as normal letters.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
     1
(*  Title:      ZF/WF.thy
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     2
    ID:         $Id$
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
     3
    Author:     Tobias Nipkow and Lawrence C Paulson
435
ca5356bd315a Addition of cardinals and order types, various tidying
lcp
parents: 124
diff changeset
     4
    Copyright   1994  University of Cambridge
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     5
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
     6
Derived first for transitive relations, and finally for arbitrary WF relations
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
     7
via wf_trancl and trans_trancl.
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
     8
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
     9
It is difficult to derive this general case directly, using r^+ instead of
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    10
r.  In is_recfun, the two occurrences of the relation must have the same
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    11
form.  Inserting r^+ in the_recfun or wftrec yields a recursion rule with
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    12
r^+ -`` {a} instead of r-``{a}.  This recursion rule is stronger in
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    13
principle, but harder to use, especially to prove wfrec_eclose_eq in
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    14
epsilon.ML.  Expanding out the definition of wftrec in wfrec would yield
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    15
a mess.
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    16
*)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    17
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13269
diff changeset
    18
header{*Well-Founded Recursion*}
c9cfe1638bf2 improved presentation markup
paulson
parents: 13269
diff changeset
    19
13357
6f54e992777e Removal of mono.thy
paulson
parents: 13356
diff changeset
    20
theory WF = Trancl:
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    21
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    22
constdefs
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    23
  wf           :: "i=>o"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    24
    (*r is a well-founded relation*)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    25
    "wf(r) == ALL Z. Z=0 | (EX x:Z. ALL y. <y,x>:r --> ~ y:Z)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    26
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    27
  wf_on        :: "[i,i]=>o"                      ("wf[_]'(_')")
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    28
    (*r is well-founded on A*)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    29
    "wf_on(A,r) == wf(r Int A*A)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    30
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    31
  is_recfun    :: "[i, i, [i,i]=>i, i] =>o"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    32
    "is_recfun(r,a,H,f) == (f = (lam x: r-``{a}. H(x, restrict(f, r-``{x}))))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    33
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    34
  the_recfun   :: "[i, i, [i,i]=>i] =>i"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    35
    "the_recfun(r,a,H) == (THE f. is_recfun(r,a,H,f))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    36
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    37
  wftrec :: "[i, i, [i,i]=>i] =>i"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    38
    "wftrec(r,a,H) == H(a, the_recfun(r,a,H))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    39
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    40
  wfrec :: "[i, i, [i,i]=>i] =>i"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    41
    (*public version.  Does not require r to be transitive*)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    42
    "wfrec(r,a,H) == wftrec(r^+, a, %x f. H(x, restrict(f,r-``{x})))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    43
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    44
  wfrec_on     :: "[i, i, i, [i,i]=>i] =>i"       ("wfrec[_]'(_,_,_')")
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    45
    "wfrec[A](r,a,H) == wfrec(r Int A*A, a, H)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    46
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    47
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13269
diff changeset
    48
subsection{*Well-Founded Relations*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    49
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
    50
subsubsection{*Equivalences between @{term wf} and @{term wf_on}*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    51
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    52
lemma wf_imp_wf_on: "wf(r) ==> wf[A](r)"
13780
af7b79271364 more new-style theories
paulson
parents: 13634
diff changeset
    53
by (unfold wf_def wf_on_def, force) 
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    54
13248
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
    55
lemma wf_on_imp_wf: "[|wf[A](r); r <= A*A|] ==> wf(r)";
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
    56
by (simp add: wf_on_def subset_Int_iff)
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
    57
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    58
lemma wf_on_field_imp_wf: "wf[field(r)](r) ==> wf(r)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    59
by (unfold wf_def wf_on_def, fast)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    60
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    61
lemma wf_iff_wf_on_field: "wf(r) <-> wf[field(r)](r)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    62
by (blast intro: wf_imp_wf_on wf_on_field_imp_wf)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    63
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    64
lemma wf_on_subset_A: "[| wf[A](r);  B<=A |] ==> wf[B](r)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    65
by (unfold wf_on_def wf_def, fast)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    66
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    67
lemma wf_on_subset_r: "[| wf[A](r); s<=r |] ==> wf[A](s)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    68
by (unfold wf_on_def wf_def, fast)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    69
13217
bc5dc2392578 new theorems
paulson
parents: 13203
diff changeset
    70
lemma wf_subset: "[|wf(s); r<=s|] ==> wf(r)"
bc5dc2392578 new theorems
paulson
parents: 13203
diff changeset
    71
by (simp add: wf_def, fast)
bc5dc2392578 new theorems
paulson
parents: 13203
diff changeset
    72
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
    73
subsubsection{*Introduction Rules for @{term wf_on}*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    74
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
    75
text{*If every non-empty subset of @{term A} has an @{term r}-minimal element
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
    76
   then we have @{term "wf[A](r)"}.*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    77
lemma wf_onI:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    78
 assumes prem: "!!Z u. [| Z<=A;  u:Z;  ALL x:Z. EX y:Z. <y,x>:r |] ==> False"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    79
 shows         "wf[A](r)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    80
apply (unfold wf_on_def wf_def)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    81
apply (rule equals0I [THEN disjCI, THEN allI])
13784
b9f6154427a4 tidying (by script)
paulson
parents: 13780
diff changeset
    82
apply (rule_tac Z = Z in prem, blast+)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    83
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    84
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
    85
text{*If @{term r} allows well-founded induction over @{term A}
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
    86
   then we have @{term "wf[A](r)"}.   Premise is equivalent to
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
    87
  @{term "!!B. ALL x:A. (ALL y. <y,x>: r --> y:B) --> x:B ==> A<=B"} *}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    88
lemma wf_onI2:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    89
 assumes prem: "!!y B. [| ALL x:A. (ALL y:A. <y,x>:r --> y:B) --> x:B;   y:A |]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    90
                       ==> y:B"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    91
 shows         "wf[A](r)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    92
apply (rule wf_onI)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    93
apply (rule_tac c=u in prem [THEN DiffE])
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    94
  prefer 3 apply blast 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    95
 apply fast+
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    96
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    97
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
    98
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
    99
subsubsection{*Well-founded Induction*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   100
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   101
text{*Consider the least @{term z} in @{term "domain(r)"} such that
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   102
  @{term "P(z)"} does not hold...*}
13534
ca6debb89d77 avoid duplicate fact bindings;
wenzelm
parents: 13357
diff changeset
   103
lemma wf_induct [induct set: wf]:
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   104
    "[| wf(r);
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   105
        !!x.[| ALL y. <y,x>: r --> P(y) |] ==> P(x) |]  
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   106
     ==> P(a)"
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   107
apply (unfold wf_def) 
13252
8c79a0dce4c0 tweaked
paulson
parents: 13248
diff changeset
   108
apply (erule_tac x = "{z : domain(r). ~ P(z)}" in allE)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   109
apply blast 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   110
done
435
ca5356bd315a Addition of cardinals and order types, various tidying
lcp
parents: 124
diff changeset
   111
13534
ca6debb89d77 avoid duplicate fact bindings;
wenzelm
parents: 13357
diff changeset
   112
lemmas wf_induct_rule = wf_induct [rule_format, induct set: wf]
13203
fac77a839aa2 Tidying up. Mainly moving proofs from Main.thy to other (Isar) theory files.
paulson
parents: 13175
diff changeset
   113
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   114
text{*The form of this rule is designed to match @{text wfI}*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   115
lemma wf_induct2:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   116
    "[| wf(r);  a:A;  field(r)<=A;
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   117
        !!x.[| x: A;  ALL y. <y,x>: r --> P(y) |] ==> P(x) |]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   118
     ==>  P(a)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   119
apply (erule_tac P="a:A" in rev_mp)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   120
apply (erule_tac a=a in wf_induct, blast) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   121
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   122
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   123
lemma field_Int_square: "field(r Int A*A) <= A"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   124
by blast
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   125
13534
ca6debb89d77 avoid duplicate fact bindings;
wenzelm
parents: 13357
diff changeset
   126
lemma wf_on_induct [consumes 2, induct set: wf_on]:
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   127
    "[| wf[A](r);  a:A;
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   128
        !!x.[| x: A;  ALL y:A. <y,x>: r --> P(y) |] ==> P(x)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   129
     |]  ==>  P(a)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   130
apply (unfold wf_on_def) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   131
apply (erule wf_induct2, assumption)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   132
apply (rule field_Int_square, blast)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   133
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   134
13534
ca6debb89d77 avoid duplicate fact bindings;
wenzelm
parents: 13357
diff changeset
   135
lemmas wf_on_induct_rule =
ca6debb89d77 avoid duplicate fact bindings;
wenzelm
parents: 13357
diff changeset
   136
  wf_on_induct [rule_format, consumes 2, induct set: wf_on]
13203
fac77a839aa2 Tidying up. Mainly moving proofs from Main.thy to other (Isar) theory files.
paulson
parents: 13175
diff changeset
   137
fac77a839aa2 Tidying up. Mainly moving proofs from Main.thy to other (Isar) theory files.
paulson
parents: 13175
diff changeset
   138
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   139
text{*If @{term r} allows well-founded induction 
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   140
   then we have @{term "wf(r)"}.*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   141
lemma wfI:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   142
    "[| field(r)<=A;
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   143
        !!y B. [| ALL x:A. (ALL y:A. <y,x>:r --> y:B) --> x:B;  y:A|]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   144
               ==> y:B |]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   145
     ==>  wf(r)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   146
apply (rule wf_on_subset_A [THEN wf_on_field_imp_wf])
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   147
apply (rule wf_onI2)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   148
 prefer 2 apply blast  
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   149
apply blast 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   150
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   151
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   152
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13269
diff changeset
   153
subsection{*Basic Properties of Well-Founded Relations*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   154
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   155
lemma wf_not_refl: "wf(r) ==> <a,a> ~: r"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   156
by (erule_tac a=a in wf_induct, blast)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   157
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   158
lemma wf_not_sym [rule_format]: "wf(r) ==> ALL x. <a,x>:r --> <x,a> ~: r"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   159
by (erule_tac a=a in wf_induct, blast)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   160
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   161
(* [| wf(r);  <a,x> : r;  ~P ==> <x,a> : r |] ==> P *)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   162
lemmas wf_asym = wf_not_sym [THEN swap, standard]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   163
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   164
lemma wf_on_not_refl: "[| wf[A](r); a: A |] ==> <a,a> ~: r"
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13252
diff changeset
   165
by (erule_tac a=a in wf_on_induct, assumption, blast)
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   166
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   167
lemma wf_on_not_sym [rule_format]:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   168
     "[| wf[A](r);  a:A |] ==> ALL b:A. <a,b>:r --> <b,a>~:r"
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13252
diff changeset
   169
apply (erule_tac a=a in wf_on_induct, assumption, blast)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   170
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   171
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   172
lemma wf_on_asym:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   173
     "[| wf[A](r);  ~Z ==> <a,b> : r;
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   174
         <b,a> ~: r ==> Z; ~Z ==> a : A; ~Z ==> b : A |] ==> Z"
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13252
diff changeset
   175
by (blast dest: wf_on_not_sym) 
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   176
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   177
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   178
(*Needed to prove well_ordI.  Could also reason that wf[A](r) means
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   179
  wf(r Int A*A);  thus wf( (r Int A*A)^+ ) and use wf_not_refl *)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   180
lemma wf_on_chain3:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   181
     "[| wf[A](r); <a,b>:r; <b,c>:r; <c,a>:r; a:A; b:A; c:A |] ==> P"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   182
apply (subgoal_tac "ALL y:A. ALL z:A. <a,y>:r --> <y,z>:r --> <z,a>:r --> P",
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   183
       blast) 
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13252
diff changeset
   184
apply (erule_tac a=a in wf_on_induct, assumption, blast)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   185
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   186
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   187
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   188
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   189
text{*transitive closure of a WF relation is WF provided 
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   190
  @{term A} is downward closed*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   191
lemma wf_on_trancl:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   192
    "[| wf[A](r);  r-``A <= A |] ==> wf[A](r^+)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   193
apply (rule wf_onI2)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   194
apply (frule bspec [THEN mp], assumption+)
13784
b9f6154427a4 tidying (by script)
paulson
parents: 13780
diff changeset
   195
apply (erule_tac a = y in wf_on_induct, assumption)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   196
apply (blast elim: tranclE, blast) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   197
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   198
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   199
lemma wf_trancl: "wf(r) ==> wf(r^+)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   200
apply (simp add: wf_iff_wf_on_field)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   201
apply (rule wf_on_subset_A) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   202
 apply (erule wf_on_trancl)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   203
 apply blast 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   204
apply (rule trancl_type [THEN field_rel_subset])
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   205
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   206
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   207
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   208
text{*@{term "r-``{a}"} is the set of everything under @{term a} in @{term r}*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   209
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   210
lemmas underI = vimage_singleton_iff [THEN iffD2, standard]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   211
lemmas underD = vimage_singleton_iff [THEN iffD1, standard]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   212
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   213
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   214
subsection{*The Predicate @{term is_recfun}*}
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   215
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   216
lemma is_recfun_type: "is_recfun(r,a,H,f) ==> f: r-``{a} -> range(f)"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   217
apply (unfold is_recfun_def)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   218
apply (erule ssubst)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   219
apply (rule lamI [THEN rangeI, THEN lam_type], assumption)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   220
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   221
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13252
diff changeset
   222
lemmas is_recfun_imp_function = is_recfun_type [THEN fun_is_function]
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13252
diff changeset
   223
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   224
lemma apply_recfun:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   225
    "[| is_recfun(r,a,H,f); <x,a>:r |] ==> f`x = H(x, restrict(f,r-``{x}))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   226
apply (unfold is_recfun_def) 
13175
81082cfa5618 new definition of "apply" and new simprule "beta_if"
paulson
parents: 13165
diff changeset
   227
  txt{*replace f only on the left-hand side*}
81082cfa5618 new definition of "apply" and new simprule "beta_if"
paulson
parents: 13165
diff changeset
   228
apply (erule_tac P = "%x.?t(x) = ?u" in ssubst)
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13252
diff changeset
   229
apply (simp add: underI) 
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   230
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   231
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   232
lemma is_recfun_equal [rule_format]:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   233
     "[| wf(r);  trans(r);  is_recfun(r,a,H,f);  is_recfun(r,b,H,g) |]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   234
      ==> <x,a>:r --> <x,b>:r --> f`x=g`x"
13784
b9f6154427a4 tidying (by script)
paulson
parents: 13780
diff changeset
   235
apply (frule_tac f = f in is_recfun_type)
b9f6154427a4 tidying (by script)
paulson
parents: 13780
diff changeset
   236
apply (frule_tac f = g in is_recfun_type)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   237
apply (simp add: is_recfun_def)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   238
apply (erule_tac a=x in wf_induct)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   239
apply (intro impI)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   240
apply (elim ssubst)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   241
apply (simp (no_asm_simp) add: vimage_singleton_iff restrict_def)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   242
apply (rule_tac t = "%z. H (?x,z) " in subst_context)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   243
apply (subgoal_tac "ALL y : r-``{x}. ALL z. <y,z>:f <-> <y,z>:g")
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   244
 apply (blast dest: transD)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   245
apply (simp add: apply_iff)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   246
apply (blast dest: transD intro: sym)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   247
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   248
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   249
lemma is_recfun_cut:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   250
     "[| wf(r);  trans(r);
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   251
         is_recfun(r,a,H,f);  is_recfun(r,b,H,g);  <b,a>:r |]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   252
      ==> restrict(f, r-``{b}) = g"
13784
b9f6154427a4 tidying (by script)
paulson
parents: 13780
diff changeset
   253
apply (frule_tac f = f in is_recfun_type)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   254
apply (rule fun_extension)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   255
  apply (blast dest: transD intro: restrict_type2)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   256
 apply (erule is_recfun_type, simp)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   257
apply (blast dest: transD intro: is_recfun_equal)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   258
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   259
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13269
diff changeset
   260
subsection{*Recursion: Main Existence Lemma*}
435
ca5356bd315a Addition of cardinals and order types, various tidying
lcp
parents: 124
diff changeset
   261
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   262
lemma is_recfun_functional:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   263
     "[| wf(r); trans(r); is_recfun(r,a,H,f); is_recfun(r,a,H,g) |]  ==>  f=g"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   264
by (blast intro: fun_extension is_recfun_type is_recfun_equal)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   265
13248
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
   266
lemma the_recfun_eq:
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
   267
    "[| is_recfun(r,a,H,f);  wf(r);  trans(r) |] ==> the_recfun(r,a,H) = f"
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
   268
apply (unfold the_recfun_def)
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
   269
apply (blast intro: is_recfun_functional)
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
   270
done
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
   271
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   272
(*If some f satisfies is_recfun(r,a,H,-) then so does the_recfun(r,a,H) *)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   273
lemma is_the_recfun:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   274
    "[| is_recfun(r,a,H,f);  wf(r);  trans(r) |]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   275
     ==> is_recfun(r, a, H, the_recfun(r,a,H))"
13248
ae66c22ed52e new theorems
paulson
parents: 13219
diff changeset
   276
by (simp add: the_recfun_eq)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   277
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   278
lemma unfold_the_recfun:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   279
     "[| wf(r);  trans(r) |] ==> is_recfun(r, a, H, the_recfun(r,a,H))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   280
apply (rule_tac a=a in wf_induct, assumption)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   281
apply (rename_tac a1) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   282
apply (rule_tac f = "lam y: r-``{a1}. wftrec (r,y,H)" in is_the_recfun)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   283
  apply typecheck
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   284
apply (unfold is_recfun_def wftrec_def)
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   285
  --{*Applying the substitution: must keep the quantified assumption!*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   286
apply (rule lam_cong [OF refl]) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   287
apply (drule underD) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   288
apply (fold is_recfun_def)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   289
apply (rule_tac t = "%z. H(?x,z)" in subst_context)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   290
apply (rule fun_extension)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   291
  apply (blast intro: is_recfun_type)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   292
 apply (rule lam_type [THEN restrict_type2])
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   293
  apply blast
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   294
 apply (blast dest: transD)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   295
apply (frule spec [THEN mp], assumption)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   296
apply (subgoal_tac "<xa,a1> : r")
13784
b9f6154427a4 tidying (by script)
paulson
parents: 13780
diff changeset
   297
 apply (drule_tac x1 = xa in spec [THEN mp], assumption)
13175
81082cfa5618 new definition of "apply" and new simprule "beta_if"
paulson
parents: 13165
diff changeset
   298
apply (simp add: vimage_singleton_iff 
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   299
                 apply_recfun is_recfun_cut)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   300
apply (blast dest: transD)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   301
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   302
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   303
13356
c9cfe1638bf2 improved presentation markup
paulson
parents: 13269
diff changeset
   304
subsection{*Unfolding @{term "wftrec(r,a,H)"}*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   305
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   306
lemma the_recfun_cut:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   307
     "[| wf(r);  trans(r);  <b,a>:r |]
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   308
      ==> restrict(the_recfun(r,a,H), r-``{b}) = the_recfun(r,b,H)"
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13252
diff changeset
   309
by (blast intro: is_recfun_cut unfold_the_recfun)
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   310
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   311
(*NOT SUITABLE FOR REWRITING: it is recursive!*)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   312
lemma wftrec:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   313
    "[| wf(r);  trans(r) |] ==>
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   314
          wftrec(r,a,H) = H(a, lam x: r-``{a}. wftrec(r,x,H))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   315
apply (unfold wftrec_def)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   316
apply (subst unfold_the_recfun [unfolded is_recfun_def])
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   317
apply (simp_all add: vimage_singleton_iff [THEN iff_sym] the_recfun_cut)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   318
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   319
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   320
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   321
subsubsection{*Removal of the Premise @{term "trans(r)"}*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   322
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   323
(*NOT SUITABLE FOR REWRITING: it is recursive!*)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   324
lemma wfrec:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   325
    "wf(r) ==> wfrec(r,a,H) = H(a, lam x:r-``{a}. wfrec(r,x,H))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   326
apply (unfold wfrec_def) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   327
apply (erule wf_trancl [THEN wftrec, THEN ssubst])
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   328
 apply (rule trans_trancl)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   329
apply (rule vimage_pair_mono [THEN restrict_lam_eq, THEN subst_context])
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   330
 apply (erule r_into_trancl)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   331
apply (rule subset_refl)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   332
done
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   333
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   334
(*This form avoids giant explosions in proofs.  NOTE USE OF == *)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   335
lemma def_wfrec:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   336
    "[| !!x. h(x)==wfrec(r,x,H);  wf(r) |] ==>
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   337
     h(a) = H(a, lam x: r-``{a}. h(x))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   338
apply simp
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   339
apply (elim wfrec) 
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   340
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   341
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   342
lemma wfrec_type:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   343
    "[| wf(r);  a:A;  field(r)<=A;
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   344
        !!x u. [| x: A;  u: Pi(r-``{x}, B) |] ==> H(x,u) : B(x)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   345
     |] ==> wfrec(r,a,H) : B(a)"
13784
b9f6154427a4 tidying (by script)
paulson
parents: 13780
diff changeset
   346
apply (rule_tac a = a in wf_induct2, assumption+)
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   347
apply (subst wfrec, assumption)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   348
apply (simp add: lam_type underD)  
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   349
done
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   350
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   351
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   352
lemma wfrec_on:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   353
 "[| wf[A](r);  a: A |] ==>
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   354
         wfrec[A](r,a,H) = H(a, lam x: (r-``{a}) Int A. wfrec[A](r,x,H))"
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   355
apply (unfold wf_on_def wfrec_on_def)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   356
apply (erule wfrec [THEN trans])
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   357
apply (simp add: vimage_Int_square cons_subset_iff)
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   358
done
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   359
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   360
text{*Minimal-element characterization of well-foundedness*}
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   361
lemma wf_eq_minimal:
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   362
     "wf(r) <-> (ALL Q x. x:Q --> (EX z:Q. ALL y. <y,z>:r --> y~:Q))"
13634
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   363
by (unfold wf_def, blast)
99a593b49b04 Re-organization of Constructible theories
paulson
parents: 13534
diff changeset
   364
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   365
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   366
ML
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   367
{*
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   368
val wf_def = thm "wf_def";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   369
val wf_on_def = thm "wf_on_def";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   370
13165
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   371
val wf_imp_wf_on = thm "wf_imp_wf_on";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   372
val wf_on_field_imp_wf = thm "wf_on_field_imp_wf";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   373
val wf_iff_wf_on_field = thm "wf_iff_wf_on_field";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   374
val wf_on_subset_A = thm "wf_on_subset_A";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   375
val wf_on_subset_r = thm "wf_on_subset_r";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   376
val wf_onI = thm "wf_onI";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   377
val wf_onI2 = thm "wf_onI2";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   378
val wf_induct = thm "wf_induct";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   379
val wf_induct2 = thm "wf_induct2";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   380
val field_Int_square = thm "field_Int_square";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   381
val wf_on_induct = thm "wf_on_induct";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   382
val wfI = thm "wfI";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   383
val wf_not_refl = thm "wf_not_refl";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   384
val wf_not_sym = thm "wf_not_sym";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   385
val wf_asym = thm "wf_asym";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   386
val wf_on_not_refl = thm "wf_on_not_refl";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   387
val wf_on_not_sym = thm "wf_on_not_sym";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   388
val wf_on_asym = thm "wf_on_asym";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   389
val wf_on_chain3 = thm "wf_on_chain3";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   390
val wf_on_trancl = thm "wf_on_trancl";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   391
val wf_trancl = thm "wf_trancl";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   392
val underI = thm "underI";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   393
val underD = thm "underD";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   394
val is_recfun_type = thm "is_recfun_type";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   395
val apply_recfun = thm "apply_recfun";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   396
val is_recfun_equal = thm "is_recfun_equal";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   397
val is_recfun_cut = thm "is_recfun_cut";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   398
val is_recfun_functional = thm "is_recfun_functional";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   399
val is_the_recfun = thm "is_the_recfun";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   400
val unfold_the_recfun = thm "unfold_the_recfun";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   401
val the_recfun_cut = thm "the_recfun_cut";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   402
val wftrec = thm "wftrec";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   403
val wfrec = thm "wfrec";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   404
val def_wfrec = thm "def_wfrec";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   405
val wfrec_type = thm "wfrec_type";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   406
val wfrec_on = thm "wfrec_on";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   407
val wf_eq_minimal = thm "wf_eq_minimal";
31d020705aff conversion of equalities and WF to Isar
paulson
parents: 3840
diff changeset
   408
*}
435
ca5356bd315a Addition of cardinals and order types, various tidying
lcp
parents: 124
diff changeset
   409
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   410
end