src/HOL/Order_Relation.thy
author wenzelm
Mon, 01 May 2017 13:03:56 +0200
changeset 65666 45d0692bb019
parent 63952 354808e9f44b
child 68484 59793df7f853
permissions -rw-r--r--
incremental download of Jenkins log files, which are also added to database;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
54552
5d57cbec0f0f moving 'Order_Relation' to 'HOL' (since it's a BNF dependency)
blanchet
parents: 54551
diff changeset
     1
(*  Title:      HOL/Order_Relation.thy
5d57cbec0f0f moving 'Order_Relation' to 'HOL' (since it's a BNF dependency)
blanchet
parents: 54551
diff changeset
     2
    Author:     Tobias Nipkow
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
     3
    Author:     Andrei Popescu, TU Muenchen
54552
5d57cbec0f0f moving 'Order_Relation' to 'HOL' (since it's a BNF dependency)
blanchet
parents: 54551
diff changeset
     4
*)
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
     5
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
     6
section \<open>Orders as Relations\<close>
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
     7
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
     8
theory Order_Relation
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
     9
imports Wfrec
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    10
begin
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    11
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    12
subsection \<open>Orders on a set\<close>
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    13
30198
922f944f03b2 name changes
nipkow
parents: 29859
diff changeset
    14
definition "preorder_on A r \<equiv> refl_on A r \<and> trans r"
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    15
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    16
definition "partial_order_on A r \<equiv> preorder_on A r \<and> antisym r"
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    17
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    18
definition "linear_order_on A r \<equiv> partial_order_on A r \<and> total_on A r"
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    19
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    20
definition "strict_linear_order_on A r \<equiv> trans r \<and> irrefl r \<and> total_on A r"
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    21
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    22
definition "well_order_on A r \<equiv> linear_order_on A r \<and> wf(r - Id)"
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    23
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    24
lemmas order_on_defs =
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    25
  preorder_on_def partial_order_on_def linear_order_on_def
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    26
  strict_linear_order_on_def well_order_on_def
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    27
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    28
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    29
lemma preorder_on_empty[simp]: "preorder_on {} {}"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    30
  by (simp add: preorder_on_def trans_def)
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    31
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    32
lemma partial_order_on_empty[simp]: "partial_order_on {} {}"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    33
  by (simp add: partial_order_on_def)
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    34
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    35
lemma lnear_order_on_empty[simp]: "linear_order_on {} {}"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    36
  by (simp add: linear_order_on_def)
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    37
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    38
lemma well_order_on_empty[simp]: "well_order_on {} {}"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    39
  by (simp add: well_order_on_def)
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    40
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    41
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    42
lemma preorder_on_converse[simp]: "preorder_on A (r\<inverse>) = preorder_on A r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    43
  by (simp add: preorder_on_def)
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    44
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    45
lemma partial_order_on_converse[simp]: "partial_order_on A (r\<inverse>) = partial_order_on A r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    46
  by (simp add: partial_order_on_def)
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    47
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    48
lemma linear_order_on_converse[simp]: "linear_order_on A (r\<inverse>) = linear_order_on A r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    49
  by (simp add: linear_order_on_def)
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    50
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    51
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    52
lemma strict_linear_order_on_diff_Id: "linear_order_on A r \<Longrightarrow> strict_linear_order_on A (r - Id)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    53
  by (simp add: order_on_defs trans_diff_Id)
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    54
63563
0bcd79da075b prefer [simp] over [iff] as [iff] break HOL-UNITY
Andreas Lochbihler
parents: 63561
diff changeset
    55
lemma linear_order_on_singleton [simp]: "linear_order_on {x} {(x, x)}"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    56
  by (simp add: order_on_defs)
63561
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    57
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    58
lemma linear_order_on_acyclic:
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    59
  assumes "linear_order_on A r"
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    60
  shows "acyclic (r - Id)"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    61
  using strict_linear_order_on_diff_Id[OF assms]
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    62
  by (auto simp add: acyclic_irrefl strict_linear_order_on_def)
63561
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    63
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    64
lemma linear_order_on_well_order_on:
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    65
  assumes "finite r"
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    66
  shows "linear_order_on A r \<longleftrightarrow> well_order_on A r"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    67
  unfolding well_order_on_def
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    68
  using assms finite_acyclic_wf[OF _ linear_order_on_acyclic, of r] by blast
63561
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
    69
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    70
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    71
subsection \<open>Orders on the field\<close>
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    72
30198
922f944f03b2 name changes
nipkow
parents: 29859
diff changeset
    73
abbreviation "Refl r \<equiv> refl_on (Field r) r"
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    74
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    75
abbreviation "Preorder r \<equiv> preorder_on (Field r) r"
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    76
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    77
abbreviation "Partial_order r \<equiv> partial_order_on (Field r) r"
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    78
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    79
abbreviation "Total r \<equiv> total_on (Field r) r"
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    80
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    81
abbreviation "Linear_order r \<equiv> linear_order_on (Field r) r"
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    82
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    83
abbreviation "Well_order r \<equiv> well_order_on (Field r) r"
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
    84
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    85
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    86
lemma subset_Image_Image_iff:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    87
  "Preorder r \<Longrightarrow> A \<subseteq> Field r \<Longrightarrow> B \<subseteq> Field r \<Longrightarrow>
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    88
    r `` A \<subseteq> r `` B \<longleftrightarrow> (\<forall>a\<in>A.\<exists>b\<in>B. (b, a) \<in> r)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    89
  apply (simp add: preorder_on_def refl_on_def Image_def subset_eq)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    90
  apply (simp only: trans_def)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    91
  apply fast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    92
  done
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    93
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    94
lemma subset_Image1_Image1_iff:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    95
  "Preorder r \<Longrightarrow> a \<in> Field r \<Longrightarrow> b \<in> Field r \<Longrightarrow> r `` {a} \<subseteq> r `` {b} \<longleftrightarrow> (b, a) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    96
  by (simp add: subset_Image_Image_iff)
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    97
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
    98
lemma Refl_antisym_eq_Image1_Image1_iff:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
    99
  assumes "Refl r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   100
    and as: "antisym r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   101
    and abf: "a \<in> Field r" "b \<in> Field r"
54552
5d57cbec0f0f moving 'Order_Relation' to 'HOL' (since it's a BNF dependency)
blanchet
parents: 54551
diff changeset
   102
  shows "r `` {a} = r `` {b} \<longleftrightarrow> a = b"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   103
    (is "?lhs \<longleftrightarrow> ?rhs")
54552
5d57cbec0f0f moving 'Order_Relation' to 'HOL' (since it's a BNF dependency)
blanchet
parents: 54551
diff changeset
   104
proof
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   105
  assume ?lhs
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   106
  then have *: "\<And>x. (a, x) \<in> r \<longleftrightarrow> (b, x) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   107
    by (simp add: set_eq_iff)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   108
  have "(a, a) \<in> r" "(b, b) \<in> r" using \<open>Refl r\<close> abf by (simp_all add: refl_on_def)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   109
  then have "(a, b) \<in> r" "(b, a) \<in> r" using *[of a] *[of b] by simp_all
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   110
  then show ?rhs
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   111
    using \<open>antisym r\<close>[unfolded antisym_def] by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   112
next
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   113
  assume ?rhs
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   114
  then show ?lhs by fast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   115
qed
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
   116
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
   117
lemma Partial_order_eq_Image1_Image1_iff:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   118
  "Partial_order r \<Longrightarrow> a \<in> Field r \<Longrightarrow> b \<in> Field r \<Longrightarrow> r `` {a} = r `` {b} \<longleftrightarrow> a = b"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   119
  by (auto simp: order_on_defs Refl_antisym_eq_Image1_Image1_iff)
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
   120
52182
57b4fdc59d3b well-order extension (by Christian Sternagel)
popescua
parents: 48750
diff changeset
   121
lemma Total_Id_Field:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   122
  assumes "Total r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   123
    and not_Id: "\<not> r \<subseteq> Id"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   124
  shows "Field r = Field (r - Id)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   125
  using mono_Field[of "r - Id" r] Diff_subset[of r Id]
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   126
proof auto
52182
57b4fdc59d3b well-order extension (by Christian Sternagel)
popescua
parents: 48750
diff changeset
   127
  fix a assume *: "a \<in> Field r"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   128
  from not_Id have "r \<noteq> {}" by fast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   129
  with not_Id obtain b and c where "b \<noteq> c \<and> (b,c) \<in> r" by auto
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   130
  then have "b \<noteq> c \<and> {b, c} \<subseteq> Field r" by (auto simp: Field_def)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   131
  with * obtain d where "d \<in> Field r" "d \<noteq> a" by auto
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   132
  with * \<open>Total r\<close> have "(a, d) \<in> r \<or> (d, a) \<in> r" by (simp add: total_on_def)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   133
  with \<open>d \<noteq> a\<close> show "a \<in> Field (r - Id)" unfolding Field_def by blast
52182
57b4fdc59d3b well-order extension (by Christian Sternagel)
popescua
parents: 48750
diff changeset
   134
qed
57b4fdc59d3b well-order extension (by Christian Sternagel)
popescua
parents: 48750
diff changeset
   135
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
   136
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   137
subsection \<open>Orders on a type\<close>
26295
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
   138
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
   139
abbreviation "strict_linear_order \<equiv> strict_linear_order_on UNIV"
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
   140
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
   141
abbreviation "linear_order \<equiv> linear_order_on UNIV"
afc43168ed85 More defns and thms
nipkow
parents: 26273
diff changeset
   142
54551
4cd6deb430c3 fixed apparent copy-paste bug
blanchet
parents: 54482
diff changeset
   143
abbreviation "well_order \<equiv> well_order_on UNIV"
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
   144
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   145
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
   146
subsection \<open>Order-like relations\<close>
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   147
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   148
text \<open>
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   149
  In this subsection, we develop basic concepts and results pertaining
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   150
  to order-like relations, i.e., to reflexive and/or transitive and/or symmetric and/or
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   151
  total relations. We also further define upper and lower bounds operators.
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   152
\<close>
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   153
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   154
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
   155
subsubsection \<open>Auxiliaries\<close>
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   156
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   157
lemma refl_on_domain: "refl_on A r \<Longrightarrow> (a, b) \<in> r \<Longrightarrow> a \<in> A \<and> b \<in> A"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   158
  by (auto simp add: refl_on_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   159
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   160
corollary well_order_on_domain: "well_order_on A r \<Longrightarrow> (a, b) \<in> r \<Longrightarrow> a \<in> A \<and> b \<in> A"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   161
  by (auto simp add: refl_on_domain order_on_defs)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   162
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   163
lemma well_order_on_Field: "well_order_on A r \<Longrightarrow> A = Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   164
  by (auto simp add: refl_on_def Field_def order_on_defs)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   165
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   166
lemma well_order_on_Well_order: "well_order_on A r \<Longrightarrow> A = Field r \<and> Well_order r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   167
  using well_order_on_Field [of A] by auto
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   168
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   169
lemma Total_subset_Id:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   170
  assumes "Total r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   171
    and "r \<subseteq> Id"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   172
  shows "r = {} \<or> (\<exists>a. r = {(a, a)})"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   173
proof -
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   174
  have "\<exists>a. r = {(a, a)}" if "r \<noteq> {}"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   175
  proof -
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   176
    from that obtain a b where ab: "(a, b) \<in> r" by fast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   177
    with \<open>r \<subseteq> Id\<close> have "a = b" by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   178
    with ab have aa: "(a, a) \<in> r" by simp
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   179
    have "a = c \<and> a = d" if "(c, d) \<in> r" for c d
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   180
    proof -
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   181
      from that have "{a, c, d} \<subseteq> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   182
        using ab unfolding Field_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   183
      then have "((a, c) \<in> r \<or> (c, a) \<in> r \<or> a = c) \<and> ((a, d) \<in> r \<or> (d, a) \<in> r \<or> a = d)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   184
        using \<open>Total r\<close> unfolding total_on_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   185
      with \<open>r \<subseteq> Id\<close> show ?thesis by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   186
    qed
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   187
    then have "r \<subseteq> {(a, a)}" by auto
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   188
    with aa show ?thesis by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   189
  qed
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   190
  then show ?thesis by blast
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   191
qed
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   192
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   193
lemma Linear_order_in_diff_Id:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   194
  assumes "Linear_order r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   195
    and "a \<in> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   196
    and "b \<in> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   197
  shows "(a, b) \<in> r \<longleftrightarrow> (b, a) \<notin> r - Id"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   198
  using assms unfolding order_on_defs total_on_def antisym_def Id_def refl_on_def by force
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   199
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   200
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
   201
subsubsection \<open>The upper and lower bounds operators\<close>
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   202
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   203
text \<open>
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   204
  Here we define upper (``above") and lower (``below") bounds operators. We
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   205
  think of \<open>r\<close> as a \<^emph>\<open>non-strict\<close> relation. The suffix \<open>S\<close> at the names of
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   206
  some operators indicates that the bounds are strict -- e.g., \<open>underS a\<close> is
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   207
  the set of all strict lower bounds of \<open>a\<close> (w.r.t. \<open>r\<close>). Capitalization of
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   208
  the first letter in the name reminds that the operator acts on sets, rather
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   209
  than on individual elements.
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   210
\<close>
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   211
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   212
definition under :: "'a rel \<Rightarrow> 'a \<Rightarrow> 'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   213
  where "under r a \<equiv> {b. (b, a) \<in> r}"
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   214
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   215
definition underS :: "'a rel \<Rightarrow> 'a \<Rightarrow> 'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   216
  where "underS r a \<equiv> {b. b \<noteq> a \<and> (b, a) \<in> r}"
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   217
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   218
definition Under :: "'a rel \<Rightarrow> 'a set \<Rightarrow> 'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   219
  where "Under r A \<equiv> {b \<in> Field r. \<forall>a \<in> A. (b, a) \<in> r}"
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   220
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   221
definition UnderS :: "'a rel \<Rightarrow> 'a set \<Rightarrow> 'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   222
  where "UnderS r A \<equiv> {b \<in> Field r. \<forall>a \<in> A. b \<noteq> a \<and> (b, a) \<in> r}"
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   223
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   224
definition above :: "'a rel \<Rightarrow> 'a \<Rightarrow> 'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   225
  where "above r a \<equiv> {b. (a, b) \<in> r}"
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   226
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   227
definition aboveS :: "'a rel \<Rightarrow> 'a \<Rightarrow> 'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   228
  where "aboveS r a \<equiv> {b. b \<noteq> a \<and> (a, b) \<in> r}"
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   229
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   230
definition Above :: "'a rel \<Rightarrow> 'a set \<Rightarrow> 'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   231
  where "Above r A \<equiv> {b \<in> Field r. \<forall>a \<in> A. (a, b) \<in> r}"
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   232
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   233
definition AboveS :: "'a rel \<Rightarrow> 'a set \<Rightarrow> 'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   234
  where "AboveS r A \<equiv> {b \<in> Field r. \<forall>a \<in> A. b \<noteq> a \<and> (a, b) \<in> r}"
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   235
55173
5556470a02b7 define ofilter outside of wo_rel
traytel
parents: 55027
diff changeset
   236
definition ofilter :: "'a rel \<Rightarrow> 'a set \<Rightarrow> bool"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   237
  where "ofilter r A \<equiv> A \<subseteq> Field r \<and> (\<forall>a \<in> A. under r a \<subseteq> A)"
55173
5556470a02b7 define ofilter outside of wo_rel
traytel
parents: 55027
diff changeset
   238
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   239
text \<open>
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   240
  Note: In the definitions of \<open>Above[S]\<close> and \<open>Under[S]\<close>, we bounded
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   241
  comprehension by \<open>Field r\<close> in order to properly cover the case of \<open>A\<close> being
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   242
  empty.
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   243
\<close>
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   244
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   245
lemma underS_subset_under: "underS r a \<subseteq> under r a"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   246
  by (auto simp add: underS_def under_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   247
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   248
lemma underS_notIn: "a \<notin> underS r a"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   249
  by (simp add: underS_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   250
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   251
lemma Refl_under_in: "Refl r \<Longrightarrow> a \<in> Field r \<Longrightarrow> a \<in> under r a"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   252
  by (simp add: refl_on_def under_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   253
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   254
lemma AboveS_disjoint: "A \<inter> (AboveS r A) = {}"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   255
  by (auto simp add: AboveS_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   256
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   257
lemma in_AboveS_underS: "a \<in> Field r \<Longrightarrow> a \<in> AboveS r (underS r a)"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   258
  by (auto simp add: AboveS_def underS_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   259
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   260
lemma Refl_under_underS: "Refl r \<Longrightarrow> a \<in> Field r \<Longrightarrow> under r a = underS r a \<union> {a}"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   261
  unfolding under_def underS_def
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   262
  using refl_on_def[of _ r] by fastforce
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   263
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   264
lemma underS_empty: "a \<notin> Field r \<Longrightarrow> underS r a = {}"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   265
  by (auto simp: Field_def underS_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   266
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   267
lemma under_Field: "under r a \<subseteq> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   268
  by (auto simp: under_def Field_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   269
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   270
lemma underS_Field: "underS r a \<subseteq> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   271
  by (auto simp: underS_def Field_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   272
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   273
lemma underS_Field2: "a \<in> Field r \<Longrightarrow> underS r a \<subset> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   274
  using underS_notIn underS_Field by fast
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   275
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   276
lemma underS_Field3: "Field r \<noteq> {} \<Longrightarrow> underS r a \<subset> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   277
  by (cases "a \<in> Field r") (auto simp: underS_Field2 underS_empty)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   278
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   279
lemma AboveS_Field: "AboveS r A \<subseteq> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   280
  by (auto simp: AboveS_def Field_def)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   281
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   282
lemma under_incr:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   283
  assumes "trans r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   284
    and "(a, b) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   285
  shows "under r a \<subseteq> under r b"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   286
  unfolding under_def
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   287
proof auto
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   288
  fix x assume "(x, a) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   289
  with assms trans_def[of r] show "(x, b) \<in> r" by blast
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   290
qed
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   291
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   292
lemma underS_incr:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   293
  assumes "trans r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   294
    and "antisym r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   295
    and ab: "(a, b) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   296
  shows "underS r a \<subseteq> underS r b"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   297
  unfolding underS_def
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   298
proof auto
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   299
  assume *: "b \<noteq> a" and **: "(b, a) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   300
  with \<open>antisym r\<close> antisym_def[of r] ab show False
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   301
    by blast
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   302
next
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   303
  fix x assume "x \<noteq> a" "(x, a) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   304
  with ab \<open>trans r\<close> trans_def[of r] show "(x, b) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   305
    by blast
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   306
qed
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   307
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   308
lemma underS_incl_iff:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   309
  assumes LO: "Linear_order r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   310
    and INa: "a \<in> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   311
    and INb: "b \<in> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   312
  shows "underS r a \<subseteq> underS r b \<longleftrightarrow> (a, b) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   313
    (is "?lhs \<longleftrightarrow> ?rhs")
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   314
proof
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   315
  assume ?rhs
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   316
  with \<open>Linear_order r\<close> show ?lhs
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   317
    by (simp add: order_on_defs underS_incr)
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   318
next
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   319
  assume *: ?lhs
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   320
  have "(a, b) \<in> r" if "a = b"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   321
    using assms that by (simp add: order_on_defs refl_on_def)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   322
  moreover have False if "a \<noteq> b" "(b, a) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   323
  proof -
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   324
    from that have "b \<in> underS r a" unfolding underS_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   325
    with * have "b \<in> underS r b" by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   326
    then show ?thesis by (simp add: underS_notIn)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   327
  qed
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   328
  ultimately show "(a,b) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   329
    using assms order_on_defs[of "Field r" r] total_on_def[of "Field r" r] by blast
55026
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   330
qed
258fa7b5a621 folded 'Order_Relation_More_FP' into 'Order_Relation'
blanchet
parents: 54552
diff changeset
   331
63561
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   332
lemma finite_Linear_order_induct[consumes 3, case_names step]:
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   333
  assumes "Linear_order r"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   334
    and "x \<in> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   335
    and "finite r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   336
    and step: "\<And>x. x \<in> Field r \<Longrightarrow> (\<And>y. y \<in> aboveS r x \<Longrightarrow> P y) \<Longrightarrow> P x"
63561
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   337
  shows "P x"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   338
  using assms(2)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   339
proof (induct rule: wf_induct[of "r\<inverse> - Id"])
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   340
  case 1
63561
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   341
  from assms(1,3) show "wf (r\<inverse> - Id)"
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   342
    using linear_order_on_well_order_on linear_order_on_converse
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   343
    unfolding well_order_on_def by blast
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   344
next
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   345
  case prems: (2 x)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   346
  show ?case
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   347
    by (rule step) (use prems in \<open>auto simp: aboveS_def intro: FieldI2\<close>)
63561
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   348
qed
fba08009ff3e add lemmas contributed by Peter Gammie
Andreas Lochbihler
parents: 61799
diff changeset
   349
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   350
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
   351
subsection \<open>Variations on Well-Founded Relations\<close>
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   352
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
   353
text \<open>
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   354
  This subsection contains some variations of the results from @{theory Wellfounded}:
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   355
    \<^item> means for slightly more direct definitions by well-founded recursion;
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   356
    \<^item> variations of well-founded induction;
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   357
    \<^item> means for proving a linear order to be a well-order.
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
   358
\<close>
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   359
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   360
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
   361
subsubsection \<open>Characterizations of well-foundedness\<close>
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   362
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   363
text \<open>
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   364
  A transitive relation is well-founded iff it is ``locally'' well-founded,
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   365
  i.e., iff its restriction to the lower bounds of of any element is
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   366
  well-founded.
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   367
\<close>
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   368
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   369
lemma trans_wf_iff:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   370
  assumes "trans r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   371
  shows "wf r \<longleftrightarrow> (\<forall>a. wf (r \<inter> (r\<inverse>``{a} \<times> r\<inverse>``{a})))"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   372
proof -
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   373
  define R where "R a = r \<inter> (r\<inverse>``{a} \<times> r\<inverse>``{a})" for a
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   374
  have "wf (R a)" if "wf r" for a
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   375
    using that R_def wf_subset[of r "R a"] by auto
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   376
  moreover
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   377
  have "wf r" if *: "\<forall>a. wf(R a)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   378
    unfolding wf_def
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   379
  proof clarify
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   380
    fix phi a
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   381
    assume **: "\<forall>a. (\<forall>b. (b, a) \<in> r \<longrightarrow> phi b) \<longrightarrow> phi a"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   382
    define chi where "chi b \<longleftrightarrow> (b, a) \<in> r \<longrightarrow> phi b" for b
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   383
    with * have "wf (R a)" by auto
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   384
    then have "(\<forall>b. (\<forall>c. (c, b) \<in> R a \<longrightarrow> chi c) \<longrightarrow> chi b) \<longrightarrow> (\<forall>b. chi b)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   385
      unfolding wf_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   386
    also have "\<forall>b. (\<forall>c. (c, b) \<in> R a \<longrightarrow> chi c) \<longrightarrow> chi b"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   387
    proof (auto simp add: chi_def R_def)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   388
      fix b
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   389
      assume "(b, a) \<in> r" and "\<forall>c. (c, b) \<in> r \<and> (c, a) \<in> r \<longrightarrow> phi c"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   390
      then have "\<forall>c. (c, b) \<in> r \<longrightarrow> phi c"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   391
        using assms trans_def[of r] by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   392
      with ** show "phi b" by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   393
    qed
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   394
    finally have  "\<forall>b. chi b" .
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   395
    with ** chi_def show "phi a" by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   396
  qed
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   397
  ultimately show ?thesis unfolding R_def by blast
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   398
qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   399
63952
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   400
text\<open>A transitive relation is well-founded if all initial segments are finite.\<close>
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   401
corollary wf_finite_segments:
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   402
  assumes "irrefl r" and "trans r" and "\<And>x. finite {y. (y, x) \<in> r}"
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   403
  shows "wf (r)"
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   404
proof (clarsimp simp: trans_wf_iff wf_iff_acyclic_if_finite converse_def assms)
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   405
  fix a
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   406
  have "trans (r \<inter> ({x. (x, a) \<in> r} \<times> {x. (x, a) \<in> r}))"
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   407
    using assms unfolding trans_def Field_def by blast
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   408
  then show "acyclic (r \<inter> {x. (x, a) \<in> r} \<times> {x. (x, a) \<in> r})"
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   409
    using assms acyclic_def assms irrefl_def by fastforce
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   410
qed
354808e9f44b new material connected with HOL Light measure theory, plus more rationalisation
paulson <lp15@cam.ac.uk>
parents: 63572
diff changeset
   411
61799
4cf66f21b764 isabelle update_cartouches -c -t;
wenzelm
parents: 60758
diff changeset
   412
text \<open>The next lemma is a variation of \<open>wf_eq_minimal\<close> from Wellfounded,
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   413
  allowing one to assume the set included in the field.\<close>
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   414
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   415
lemma wf_eq_minimal2: "wf r \<longleftrightarrow> (\<forall>A. A \<subseteq> Field r \<and> A \<noteq> {} \<longrightarrow> (\<exists>a \<in> A. \<forall>a' \<in> A. (a', a) \<notin> r))"
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   416
proof-
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   417
  let ?phi = "\<lambda>A. A \<noteq> {} \<longrightarrow> (\<exists>a \<in> A. \<forall>a' \<in> A. (a',a) \<notin> r)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   418
  have "wf r \<longleftrightarrow> (\<forall>A. ?phi A)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   419
    apply (auto simp: ex_in_conv [THEN sym])
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   420
     apply (erule wfE_min)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   421
      apply assumption
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   422
     apply blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   423
    apply (rule wfI_min)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   424
    apply fast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   425
    done
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   426
  also have "(\<forall>A. ?phi A) \<longleftrightarrow> (\<forall>B \<subseteq> Field r. ?phi B)"
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   427
  proof
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   428
    assume "\<forall>A. ?phi A"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   429
    then show "\<forall>B \<subseteq> Field r. ?phi B" by simp
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   430
  next
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   431
    assume *: "\<forall>B \<subseteq> Field r. ?phi B"
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   432
    show "\<forall>A. ?phi A"
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   433
    proof clarify
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   434
      fix A :: "'a set"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   435
      assume **: "A \<noteq> {}"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   436
      define B where "B = A \<inter> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   437
      show "\<exists>a \<in> A. \<forall>a' \<in> A. (a', a) \<notin> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   438
      proof (cases "B = {}")
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   439
        case True
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   440
        with ** obtain a where a: "a \<in> A" "a \<notin> Field r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   441
          unfolding B_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   442
        with a have "\<forall>a' \<in> A. (a',a) \<notin> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   443
          unfolding Field_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   444
        with a show ?thesis by blast
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   445
      next
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   446
        case False
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   447
        have "B \<subseteq> Field r" unfolding B_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   448
        with False * obtain a where a: "a \<in> B" "\<forall>a' \<in> B. (a', a) \<notin> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   449
          by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   450
        have "(a', a) \<notin> r" if "a' \<in> A" for a'
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   451
        proof
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   452
          assume a'a: "(a', a) \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   453
          with that have "a' \<in> B" unfolding B_def Field_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   454
          with a a'a show False by blast
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   455
        qed
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   456
        with a show ?thesis unfolding B_def by blast
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   457
      qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   458
    qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   459
  qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   460
  finally show ?thesis by blast
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   461
qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   462
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   463
60758
d8d85a8172b5 isabelle update_cartouches;
wenzelm
parents: 58889
diff changeset
   464
subsubsection \<open>Characterizations of well-foundedness\<close>
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   465
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   466
text \<open>
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   467
  The next lemma and its corollary enable one to prove that a linear order is
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   468
  a well-order in a way which is more standard than via well-foundedness of
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   469
  the strict version of the relation.
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   470
\<close>
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   471
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   472
lemma Linear_order_wf_diff_Id:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   473
  assumes "Linear_order r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   474
  shows "wf (r - Id) \<longleftrightarrow> (\<forall>A \<subseteq> Field r. A \<noteq> {} \<longrightarrow> (\<exists>a \<in> A. \<forall>a' \<in> A. (a, a') \<in> r))"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   475
proof (cases "r \<subseteq> Id")
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   476
  case True
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   477
  then have *: "r - Id = {}" by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   478
  have "wf (r - Id)" by (simp add: *)
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   479
  moreover have "\<exists>a \<in> A. \<forall>a' \<in> A. (a, a') \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   480
    if *: "A \<subseteq> Field r" and **: "A \<noteq> {}" for A
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   481
  proof -
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   482
    from \<open>Linear_order r\<close> True
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   483
    obtain a where a: "r = {} \<or> r = {(a, a)}"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   484
      unfolding order_on_defs using Total_subset_Id [of r] by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   485
    with * ** have "A = {a} \<and> r = {(a, a)}"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   486
      unfolding Field_def by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   487
    with a show ?thesis by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   488
  qed
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   489
  ultimately show ?thesis by blast
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   490
next
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   491
  case False
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   492
  with \<open>Linear_order r\<close> have Field: "Field r = Field (r - Id)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   493
    unfolding order_on_defs using Total_Id_Field [of r] by blast
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   494
  show ?thesis
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   495
  proof
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   496
    assume *: "wf (r - Id)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   497
    show "\<forall>A \<subseteq> Field r. A \<noteq> {} \<longrightarrow> (\<exists>a \<in> A. \<forall>a' \<in> A. (a, a') \<in> r)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   498
    proof clarify
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   499
      fix A
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   500
      assume **: "A \<subseteq> Field r" and ***: "A \<noteq> {}"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   501
      then have "\<exists>a \<in> A. \<forall>a' \<in> A. (a',a) \<notin> r - Id"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   502
        using Field * unfolding wf_eq_minimal2 by simp
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   503
      moreover have "\<forall>a \<in> A. \<forall>a' \<in> A. (a, a') \<in> r \<longleftrightarrow> (a', a) \<notin> r - Id"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   504
        using Linear_order_in_diff_Id [OF \<open>Linear_order r\<close>] ** by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   505
      ultimately show "\<exists>a \<in> A. \<forall>a' \<in> A. (a, a') \<in> r" by blast
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   506
    qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   507
  next
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   508
    assume *: "\<forall>A \<subseteq> Field r. A \<noteq> {} \<longrightarrow> (\<exists>a \<in> A. \<forall>a' \<in> A. (a, a') \<in> r)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   509
    show "wf (r - Id)"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   510
      unfolding wf_eq_minimal2
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   511
    proof clarify
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   512
      fix A
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   513
      assume **: "A \<subseteq> Field(r - Id)" and ***: "A \<noteq> {}"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   514
      then have "\<exists>a \<in> A. \<forall>a' \<in> A. (a,a') \<in> r"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   515
        using Field * by simp
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   516
      moreover have "\<forall>a \<in> A. \<forall>a' \<in> A. (a, a') \<in> r \<longleftrightarrow> (a', a) \<notin> r - Id"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   517
        using Linear_order_in_diff_Id [OF \<open>Linear_order r\<close>] ** mono_Field[of "r - Id" r] by blast
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   518
      ultimately show "\<exists>a \<in> A. \<forall>a' \<in> A. (a',a) \<notin> r - Id"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   519
        by blast
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   520
    qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   521
  qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   522
qed
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   523
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   524
corollary Linear_order_Well_order_iff:
63572
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   525
  "Linear_order r \<Longrightarrow>
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   526
    Well_order r \<longleftrightarrow> (\<forall>A \<subseteq> Field r. A \<noteq> {} \<longrightarrow> (\<exists>a \<in> A. \<forall>a' \<in> A. (a, a') \<in> r))"
c0cbfd2b5a45 misc tuning and modernization;
wenzelm
parents: 63563
diff changeset
   527
  unfolding well_order_on_def using Linear_order_wf_diff_Id[of r] by blast
55027
a74ea6d75571 folded 'Wellfounded_More_FP' into 'Wellfounded'
blanchet
parents: 55026
diff changeset
   528
26273
6c4d534af98d Orders as relations
nipkow
parents:
diff changeset
   529
end