src/HOL/Nitpick_Examples/Manual_Nits.thy
author blanchet
Wed, 21 Apr 2010 14:46:29 +0200
changeset 36268 65aabc2c89ae
parent 35738 c910fe606829
child 37452 e482320bcbfe
permissions -rw-r--r--
use only one thread in "Manual_Nits";
the second thread isn't helping much, and might very well be the cause of the Cygwin Isatest failure
blanchet@33197
     1
(*  Title:      HOL/Nitpick_Examples/Manual_Nits.thy
blanchet@33197
     2
    Author:     Jasmin Blanchette, TU Muenchen
blanchet@35073
     3
    Copyright   2009, 2010
blanchet@33197
     4
blanchet@33197
     5
Examples from the Nitpick manual.
blanchet@33197
     6
*)
blanchet@33197
     7
blanchet@33197
     8
header {* Examples from the Nitpick Manual *}
blanchet@33197
     9
blanchet@33197
    10
theory Manual_Nits
blanchet@35665
    11
imports Main Quotient_Product RealDef
blanchet@33197
    12
begin
blanchet@33197
    13
blanchet@33197
    14
chapter {* 3. First Steps *}
blanchet@33197
    15
blanchet@35710
    16
nitpick_params [sat_solver = MiniSat_JNI, max_threads = 1]
blanchet@33197
    17
blanchet@33197
    18
subsection {* 3.1. Propositional Logic *}
blanchet@33197
    19
blanchet@33197
    20
lemma "P \<longleftrightarrow> Q"
blanchet@35666
    21
nitpick [expect = genuine]
blanchet@33197
    22
apply auto
blanchet@35666
    23
nitpick [expect = genuine] 1
blanchet@35666
    24
nitpick [expect = genuine] 2
blanchet@33197
    25
oops
blanchet@33197
    26
blanchet@33197
    27
subsection {* 3.2. Type Variables *}
blanchet@33197
    28
blanchet@33197
    29
lemma "P x \<Longrightarrow> P (THE y. P y)"
blanchet@35666
    30
nitpick [verbose, expect = genuine]
blanchet@33197
    31
oops
blanchet@33197
    32
blanchet@33197
    33
subsection {* 3.3. Constants *}
blanchet@33197
    34
blanchet@33197
    35
lemma "P x \<Longrightarrow> P (THE y. P y)"
blanchet@35666
    36
nitpick [show_consts, expect = genuine]
blanchet@35666
    37
nitpick [full_descrs, show_consts, expect = genuine]
blanchet@35666
    38
nitpick [dont_specialize, full_descrs, show_consts, expect = genuine]
blanchet@33197
    39
oops
blanchet@33197
    40
blanchet@33197
    41
lemma "\<exists>!x. P x \<Longrightarrow> P (THE y. P y)"
blanchet@35666
    42
nitpick [expect = none]
blanchet@35666
    43
nitpick [card 'a = 1\<midarrow>50, expect = none]
blanchet@33197
    44
(* sledgehammer *)
blanchet@33197
    45
apply (metis the_equality)
blanchet@33197
    46
done
blanchet@33197
    47
blanchet@33197
    48
subsection {* 3.4. Skolemization *}
blanchet@33197
    49
blanchet@33197
    50
lemma "\<exists>g. \<forall>x. g (f x) = x \<Longrightarrow> \<forall>y. \<exists>x. y = f x"
blanchet@35666
    51
nitpick [expect = genuine]
blanchet@33197
    52
oops
blanchet@33197
    53
blanchet@33197
    54
lemma "\<exists>x. \<forall>f. f x = x"
blanchet@35666
    55
nitpick [expect = genuine]
blanchet@33197
    56
oops
blanchet@33197
    57
blanchet@33197
    58
lemma "refl r \<Longrightarrow> sym r"
blanchet@35666
    59
nitpick [expect = genuine]
blanchet@33197
    60
oops
blanchet@33197
    61
blanchet@34123
    62
subsection {* 3.5. Natural Numbers and Integers *}
blanchet@33197
    63
blanchet@33197
    64
lemma "\<lbrakk>i \<le> j; n \<le> (m\<Colon>int)\<rbrakk> \<Longrightarrow> i * n + j * m \<le> i * m + j * n"
blanchet@35666
    65
nitpick [expect = genuine]
blanchet@33197
    66
oops
blanchet@33197
    67
blanchet@33197
    68
lemma "\<forall>n. Suc n \<noteq> n \<Longrightarrow> P"
blanchet@35666
    69
nitpick [card nat = 100, check_potential, expect = genuine]
blanchet@33197
    70
oops
blanchet@33197
    71
blanchet@33197
    72
lemma "P Suc"
blanchet@35666
    73
nitpick [expect = none]
blanchet@33197
    74
oops
blanchet@33197
    75
blanchet@33197
    76
lemma "P (op +\<Colon>nat\<Rightarrow>nat\<Rightarrow>nat)"
blanchet@35666
    77
nitpick [card nat = 1, expect = genuine]
blanchet@35666
    78
nitpick [card nat = 2, expect = none]
blanchet@33197
    79
oops
blanchet@33197
    80
blanchet@33197
    81
subsection {* 3.6. Inductive Datatypes *}
blanchet@33197
    82
blanchet@33197
    83
lemma "hd (xs @ [y, y]) = hd xs"
blanchet@35666
    84
nitpick [expect = genuine]
blanchet@35666
    85
nitpick [show_consts, show_datatypes, expect = genuine]
blanchet@33197
    86
oops
blanchet@33197
    87
blanchet@33197
    88
lemma "\<lbrakk>length xs = 1; length ys = 1\<rbrakk> \<Longrightarrow> xs = ys"
blanchet@35666
    89
nitpick [show_datatypes, expect = genuine]
blanchet@33197
    90
oops
blanchet@33197
    91
blanchet@33197
    92
subsection {* 3.7. Typedefs, Records, Rationals, and Reals *}
blanchet@33197
    93
blanchet@33197
    94
typedef three = "{0\<Colon>nat, 1, 2}"
blanchet@33197
    95
by blast
blanchet@33197
    96
blanchet@33197
    97
definition A :: three where "A \<equiv> Abs_three 0"
blanchet@33197
    98
definition B :: three where "B \<equiv> Abs_three 1"
blanchet@33197
    99
definition C :: three where "C \<equiv> Abs_three 2"
blanchet@33197
   100
blanchet@33197
   101
lemma "\<lbrakk>P A; P B\<rbrakk> \<Longrightarrow> P x"
blanchet@35666
   102
nitpick [show_datatypes, expect = genuine]
blanchet@33197
   103
oops
blanchet@33197
   104
blanchet@35284
   105
fun my_int_rel where
blanchet@35284
   106
"my_int_rel (x, y) (u, v) = (x + v = u + y)"
blanchet@35284
   107
blanchet@35284
   108
quotient_type my_int = "nat \<times> nat" / my_int_rel
blanchet@35284
   109
by (auto simp add: equivp_def expand_fun_eq)
blanchet@35284
   110
blanchet@35284
   111
definition add_raw where
blanchet@35284
   112
"add_raw \<equiv> \<lambda>(x, y) (u, v). (x + (u\<Colon>nat), y + (v\<Colon>nat))"
blanchet@35284
   113
blanchet@35284
   114
quotient_definition "add\<Colon>my_int \<Rightarrow> my_int \<Rightarrow> my_int" is add_raw
blanchet@35284
   115
blanchet@35284
   116
lemma "add x y = add x x"
blanchet@35666
   117
nitpick [show_datatypes, expect = genuine]
blanchet@35284
   118
oops
blanchet@35284
   119
blanchet@35711
   120
ML {*
blanchet@35712
   121
(* Proof.context -> string -> (typ -> term list) -> typ -> term -> term *)
blanchet@35712
   122
fun my_int_postproc _ _ _ T (Const _ $ (Const _ $ t1 $ t2)) =
blanchet@35712
   123
    HOLogic.mk_number T (snd (HOLogic.dest_number t1)
blanchet@35712
   124
                         - snd (HOLogic.dest_number t2))
blanchet@35712
   125
  | my_int_postproc _ _ _ _ t = t
blanchet@35711
   126
*}
blanchet@35711
   127
blanchet@35711
   128
setup {* Nitpick.register_term_postprocessor @{typ my_int} my_int_postproc *}
blanchet@35711
   129
blanchet@35711
   130
lemma "add x y = add x x"
blanchet@35711
   131
nitpick [show_datatypes]
blanchet@35711
   132
oops
blanchet@35711
   133
blanchet@33197
   134
record point =
blanchet@33197
   135
  Xcoord :: int
blanchet@33197
   136
  Ycoord :: int
blanchet@33197
   137
blanchet@33197
   138
lemma "Xcoord (p\<Colon>point) = Xcoord (q\<Colon>point)"
blanchet@35666
   139
nitpick [show_datatypes, expect = genuine]
blanchet@33197
   140
oops
blanchet@33197
   141
blanchet@33197
   142
lemma "4 * x + 3 * (y\<Colon>real) \<noteq> 1 / 2"
blanchet@35666
   143
nitpick [show_datatypes, expect = genuine]
blanchet@33197
   144
oops
blanchet@33197
   145
blanchet@33197
   146
subsection {* 3.8. Inductive and Coinductive Predicates *}
blanchet@33197
   147
blanchet@33197
   148
inductive even where
blanchet@33197
   149
"even 0" |
blanchet@33197
   150
"even n \<Longrightarrow> even (Suc (Suc n))"
blanchet@33197
   151
blanchet@33197
   152
lemma "\<exists>n. even n \<and> even (Suc n)"
blanchet@35710
   153
nitpick [card nat = 50, unary_ints, verbose, expect = potential]
blanchet@33197
   154
oops
blanchet@33197
   155
blanchet@35710
   156
lemma "\<exists>n \<le> 49. even n \<and> even (Suc n)"
blanchet@35710
   157
nitpick [card nat = 50, unary_ints, verbose, expect = genuine]
blanchet@33197
   158
oops
blanchet@33197
   159
blanchet@33197
   160
inductive even' where
blanchet@33197
   161
"even' (0\<Colon>nat)" |
blanchet@33197
   162
"even' 2" |
blanchet@33197
   163
"\<lbrakk>even' m; even' n\<rbrakk> \<Longrightarrow> even' (m + n)"
blanchet@33197
   164
blanchet@33197
   165
lemma "\<exists>n \<in> {0, 2, 4, 6, 8}. \<not> even' n"
blanchet@35666
   166
nitpick [card nat = 10, unary_ints, verbose, show_consts, expect = genuine]
blanchet@33197
   167
oops
blanchet@33197
   168
blanchet@33197
   169
lemma "even' (n - 2) \<Longrightarrow> even' n"
blanchet@35666
   170
nitpick [card nat = 10, show_consts, expect = genuine]
blanchet@33197
   171
oops
blanchet@33197
   172
blanchet@33197
   173
coinductive nats where
blanchet@33197
   174
"nats (x\<Colon>nat) \<Longrightarrow> nats x"
blanchet@33197
   175
blanchet@33197
   176
lemma "nats = {0, 1, 2, 3, 4}"
blanchet@35666
   177
nitpick [card nat = 10, show_consts, expect = genuine]
blanchet@33197
   178
oops
blanchet@33197
   179
blanchet@33197
   180
inductive odd where
blanchet@33197
   181
"odd 1" |
blanchet@33197
   182
"\<lbrakk>odd m; even n\<rbrakk> \<Longrightarrow> odd (m + n)"
blanchet@33197
   183
blanchet@33197
   184
lemma "odd n \<Longrightarrow> odd (n - 2)"
blanchet@35666
   185
nitpick [card nat = 10, show_consts, expect = genuine]
blanchet@33197
   186
oops
blanchet@33197
   187
blanchet@33197
   188
subsection {* 3.9. Coinductive Datatypes *}
blanchet@33197
   189
blanchet@35665
   190
(* Lazy lists are defined in Andreas Lochbihler's "Coinductive" AFP entry. Since
blanchet@35665
   191
we cannot rely on its presence, we expediently provide our own axiomatization.
blanchet@35665
   192
The examples also work unchanged with Lochbihler's "Coinductive_List" theory. *)
blanchet@35665
   193
blanchet@35665
   194
typedef 'a llist = "UNIV\<Colon>('a list + (nat \<Rightarrow> 'a)) set" by auto
blanchet@35665
   195
blanchet@35666
   196
definition LNil where
blanchet@35666
   197
"LNil = Abs_llist (Inl [])"
blanchet@35665
   198
definition LCons where
blanchet@35665
   199
"LCons y ys = Abs_llist (case Rep_llist ys of
blanchet@35665
   200
                           Inl ys' \<Rightarrow> Inl (y # ys')
blanchet@35665
   201
                         | Inr f \<Rightarrow> Inr (\<lambda>n. case n of 0 \<Rightarrow> y | Suc m \<Rightarrow> f m))"
blanchet@35665
   202
blanchet@35665
   203
axiomatization iterates :: "('a \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a llist"
blanchet@35665
   204
blanchet@35665
   205
lemma iterates_def [nitpick_simp]:
blanchet@35665
   206
"iterates f a = LCons a (iterates f (f a))"
blanchet@35665
   207
sorry
blanchet@35665
   208
blanchet@35665
   209
setup {*
blanchet@35665
   210
Nitpick.register_codatatype @{typ "'a llist"} ""
blanchet@35665
   211
    (map dest_Const [@{term LNil}, @{term LCons}])
blanchet@35665
   212
*}
blanchet@35665
   213
blanchet@33197
   214
lemma "xs \<noteq> LCons a xs"
blanchet@35666
   215
nitpick [expect = genuine]
blanchet@33197
   216
oops
blanchet@33197
   217
blanchet@33197
   218
lemma "\<lbrakk>xs = LCons a xs; ys = iterates (\<lambda>b. a) b\<rbrakk> \<Longrightarrow> xs = ys"
blanchet@35666
   219
nitpick [verbose, expect = genuine]
blanchet@33197
   220
oops
blanchet@33197
   221
blanchet@33197
   222
lemma "\<lbrakk>xs = LCons a xs; ys = LCons a ys\<rbrakk> \<Longrightarrow> xs = ys"
blanchet@35666
   223
nitpick [bisim_depth = -1, show_datatypes, expect = quasi_genuine]
blanchet@35666
   224
nitpick [expect = none]
blanchet@33197
   225
sorry
blanchet@33197
   226
blanchet@33197
   227
subsection {* 3.10. Boxing *}
blanchet@33197
   228
blanchet@33197
   229
datatype tm = Var nat | Lam tm | App tm tm
blanchet@33197
   230
blanchet@33197
   231
primrec lift where
blanchet@33197
   232
"lift (Var j) k = Var (if j < k then j else j + 1)" |
blanchet@33197
   233
"lift (Lam t) k = Lam (lift t (k + 1))" |
blanchet@33197
   234
"lift (App t u) k = App (lift t k) (lift u k)"
blanchet@33197
   235
blanchet@33197
   236
primrec loose where
blanchet@33197
   237
"loose (Var j) k = (j \<ge> k)" |
blanchet@33197
   238
"loose (Lam t) k = loose t (Suc k)" |
blanchet@33197
   239
"loose (App t u) k = (loose t k \<or> loose u k)"
blanchet@33197
   240
blanchet@33197
   241
primrec subst\<^isub>1 where
blanchet@33197
   242
"subst\<^isub>1 \<sigma> (Var j) = \<sigma> j" |
blanchet@33197
   243
"subst\<^isub>1 \<sigma> (Lam t) =
blanchet@33197
   244
 Lam (subst\<^isub>1 (\<lambda>n. case n of 0 \<Rightarrow> Var 0 | Suc m \<Rightarrow> lift (\<sigma> m) 1) t)" |
blanchet@33197
   245
"subst\<^isub>1 \<sigma> (App t u) = App (subst\<^isub>1 \<sigma> t) (subst\<^isub>1 \<sigma> u)"
blanchet@33197
   246
blanchet@33197
   247
lemma "\<not> loose t 0 \<Longrightarrow> subst\<^isub>1 \<sigma> t = t"
blanchet@35666
   248
nitpick [verbose, expect = genuine]
blanchet@35666
   249
nitpick [eval = "subst\<^isub>1 \<sigma> t", expect = genuine]
blanchet@35666
   250
(* nitpick [dont_box, expect = unknown] *)
blanchet@33197
   251
oops
blanchet@33197
   252
blanchet@33197
   253
primrec subst\<^isub>2 where
blanchet@33197
   254
"subst\<^isub>2 \<sigma> (Var j) = \<sigma> j" |
blanchet@33197
   255
"subst\<^isub>2 \<sigma> (Lam t) =
blanchet@33197
   256
 Lam (subst\<^isub>2 (\<lambda>n. case n of 0 \<Rightarrow> Var 0 | Suc m \<Rightarrow> lift (\<sigma> m) 0) t)" |
blanchet@33197
   257
"subst\<^isub>2 \<sigma> (App t u) = App (subst\<^isub>2 \<sigma> t) (subst\<^isub>2 \<sigma> u)"
blanchet@33197
   258
blanchet@33197
   259
lemma "\<not> loose t 0 \<Longrightarrow> subst\<^isub>2 \<sigma> t = t"
blanchet@35710
   260
nitpick [card = 1\<midarrow>5, expect = none]
blanchet@33197
   261
sorry
blanchet@33197
   262
blanchet@33197
   263
subsection {* 3.11. Scope Monotonicity *}
blanchet@33197
   264
blanchet@33197
   265
lemma "length xs = length ys \<Longrightarrow> rev (zip xs ys) = zip xs (rev ys)"
blanchet@35666
   266
nitpick [verbose, expect = genuine]
blanchet@35666
   267
nitpick [card = 8, verbose, expect = genuine]
blanchet@33197
   268
oops
blanchet@33197
   269
blanchet@33197
   270
lemma "\<exists>g. \<forall>x\<Colon>'b. g (f x) = x \<Longrightarrow> \<forall>y\<Colon>'a. \<exists>x. y = f x"
blanchet@35666
   271
nitpick [mono, expect = none]
blanchet@35666
   272
nitpick [expect = genuine]
blanchet@33197
   273
oops
blanchet@33197
   274
blanchet@34969
   275
subsection {* 3.12. Inductive Properties *}
blanchet@34969
   276
blanchet@34969
   277
inductive_set reach where
blanchet@34969
   278
"(4\<Colon>nat) \<in> reach" |
blanchet@34969
   279
"n \<in> reach \<Longrightarrow> n < 4 \<Longrightarrow> 3 * n + 1 \<in> reach" |
blanchet@34969
   280
"n \<in> reach \<Longrightarrow> n + 2 \<in> reach"
blanchet@34969
   281
blanchet@34969
   282
lemma "n \<in> reach \<Longrightarrow> 2 dvd n"
blanchet@35714
   283
nitpick [card = 1\<midarrow>5, bits = 1\<midarrow>5, expect = none]
blanchet@34969
   284
apply (induct set: reach)
blanchet@34969
   285
  apply auto
blanchet@35714
   286
 nitpick [card = 1\<midarrow>5, bits = 1\<midarrow>5, expect = none]
blanchet@34969
   287
 apply (thin_tac "n \<in> reach")
blanchet@35666
   288
 nitpick [expect = genuine]
blanchet@34969
   289
oops
blanchet@34969
   290
blanchet@34969
   291
lemma "n \<in> reach \<Longrightarrow> 2 dvd n \<and> n \<noteq> 0"
blanchet@35714
   292
nitpick [card = 1\<midarrow>5, bits = 1\<midarrow>5, expect = none]
blanchet@34969
   293
apply (induct set: reach)
blanchet@34969
   294
  apply auto
blanchet@35714
   295
 nitpick [card = 1\<midarrow>5, bits = 1\<midarrow>5, expect = none]
blanchet@34969
   296
 apply (thin_tac "n \<in> reach")
blanchet@35666
   297
 nitpick [expect = genuine]
blanchet@34969
   298
oops
blanchet@34969
   299
blanchet@34969
   300
lemma "n \<in> reach \<Longrightarrow> 2 dvd n \<and> n \<ge> 4"
blanchet@34969
   301
by (induct set: reach) arith+
blanchet@34969
   302
blanchet@34969
   303
datatype 'a bin_tree = Leaf 'a | Branch "'a bin_tree" "'a bin_tree"
blanchet@34969
   304
blanchet@34969
   305
primrec labels where
blanchet@34969
   306
"labels (Leaf a) = {a}" |
blanchet@34969
   307
"labels (Branch t u) = labels t \<union> labels u"
blanchet@34969
   308
blanchet@34969
   309
primrec swap where
blanchet@34969
   310
"swap (Leaf c) a b =
blanchet@34969
   311
 (if c = a then Leaf b else if c = b then Leaf a else Leaf c)" |
blanchet@34969
   312
"swap (Branch t u) a b = Branch (swap t a b) (swap u a b)"
blanchet@34969
   313
blanchet@35180
   314
lemma "{a, b} \<subseteq> labels t \<Longrightarrow> labels (swap t a b) = labels t"
blanchet@35666
   315
(* nitpick *)
blanchet@34969
   316
proof (induct t)
blanchet@34969
   317
  case Leaf thus ?case by simp
blanchet@34969
   318
next
blanchet@34969
   319
  case (Branch t u) thus ?case
blanchet@35666
   320
  (* nitpick *)
blanchet@35666
   321
  nitpick [non_std, show_all, expect = genuine]
blanchet@34969
   322
oops
blanchet@34969
   323
blanchet@34969
   324
lemma "labels (swap t a b) =
blanchet@34969
   325
       (if a \<in> labels t then
blanchet@34969
   326
          if b \<in> labels t then labels t else (labels t - {a}) \<union> {b}
blanchet@34969
   327
        else
blanchet@34969
   328
          if b \<in> labels t then (labels t - {b}) \<union> {a} else labels t)"
blanchet@35309
   329
(* nitpick *)
blanchet@34969
   330
proof (induct t)
blanchet@34969
   331
  case Leaf thus ?case by simp
blanchet@34969
   332
next
blanchet@34969
   333
  case (Branch t u) thus ?case
blanchet@35710
   334
  nitpick [non_std, card = 1\<midarrow>5, expect = none]
blanchet@34969
   335
  by auto
blanchet@34969
   336
qed
blanchet@34969
   337
blanchet@33197
   338
section {* 4. Case Studies *}
blanchet@33197
   339
blanchet@36268
   340
nitpick_params [max_potential = 0]
blanchet@33197
   341
blanchet@33197
   342
subsection {* 4.1. A Context-Free Grammar *}
blanchet@33197
   343
blanchet@33197
   344
datatype alphabet = a | b
blanchet@33197
   345
blanchet@33197
   346
inductive_set S\<^isub>1 and A\<^isub>1 and B\<^isub>1 where
blanchet@33197
   347
  "[] \<in> S\<^isub>1"
blanchet@33197
   348
| "w \<in> A\<^isub>1 \<Longrightarrow> b # w \<in> S\<^isub>1"
blanchet@33197
   349
| "w \<in> B\<^isub>1 \<Longrightarrow> a # w \<in> S\<^isub>1"
blanchet@33197
   350
| "w \<in> S\<^isub>1 \<Longrightarrow> a # w \<in> A\<^isub>1"
blanchet@33197
   351
| "w \<in> S\<^isub>1 \<Longrightarrow> b # w \<in> S\<^isub>1"
blanchet@33197
   352
| "\<lbrakk>v \<in> B\<^isub>1; v \<in> B\<^isub>1\<rbrakk> \<Longrightarrow> a # v @ w \<in> B\<^isub>1"
blanchet@33197
   353
blanchet@33197
   354
theorem S\<^isub>1_sound:
blanchet@33197
   355
"w \<in> S\<^isub>1 \<longrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b]"
blanchet@35666
   356
nitpick [expect = genuine]
blanchet@33197
   357
oops
blanchet@33197
   358
blanchet@33197
   359
inductive_set S\<^isub>2 and A\<^isub>2 and B\<^isub>2 where
blanchet@33197
   360
  "[] \<in> S\<^isub>2"
blanchet@33197
   361
| "w \<in> A\<^isub>2 \<Longrightarrow> b # w \<in> S\<^isub>2"
blanchet@33197
   362
| "w \<in> B\<^isub>2 \<Longrightarrow> a # w \<in> S\<^isub>2"
blanchet@33197
   363
| "w \<in> S\<^isub>2 \<Longrightarrow> a # w \<in> A\<^isub>2"
blanchet@33197
   364
| "w \<in> S\<^isub>2 \<Longrightarrow> b # w \<in> B\<^isub>2"
blanchet@33197
   365
| "\<lbrakk>v \<in> B\<^isub>2; v \<in> B\<^isub>2\<rbrakk> \<Longrightarrow> a # v @ w \<in> B\<^isub>2"
blanchet@33197
   366
blanchet@33197
   367
theorem S\<^isub>2_sound:
blanchet@33197
   368
"w \<in> S\<^isub>2 \<longrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b]"
blanchet@35666
   369
nitpick [expect = genuine]
blanchet@33197
   370
oops
blanchet@33197
   371
blanchet@33197
   372
inductive_set S\<^isub>3 and A\<^isub>3 and B\<^isub>3 where
blanchet@33197
   373
  "[] \<in> S\<^isub>3"
blanchet@33197
   374
| "w \<in> A\<^isub>3 \<Longrightarrow> b # w \<in> S\<^isub>3"
blanchet@33197
   375
| "w \<in> B\<^isub>3 \<Longrightarrow> a # w \<in> S\<^isub>3"
blanchet@33197
   376
| "w \<in> S\<^isub>3 \<Longrightarrow> a # w \<in> A\<^isub>3"
blanchet@33197
   377
| "w \<in> S\<^isub>3 \<Longrightarrow> b # w \<in> B\<^isub>3"
blanchet@33197
   378
| "\<lbrakk>v \<in> B\<^isub>3; w \<in> B\<^isub>3\<rbrakk> \<Longrightarrow> a # v @ w \<in> B\<^isub>3"
blanchet@33197
   379
blanchet@33197
   380
theorem S\<^isub>3_sound:
blanchet@33197
   381
"w \<in> S\<^isub>3 \<longrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b]"
blanchet@35710
   382
nitpick [card = 1\<midarrow>6, expect = none]
blanchet@33197
   383
sorry
blanchet@33197
   384
blanchet@33197
   385
theorem S\<^isub>3_complete:
blanchet@33197
   386
"length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b] \<longrightarrow> w \<in> S\<^isub>3"
blanchet@35666
   387
nitpick [expect = genuine]
blanchet@33197
   388
oops
blanchet@33197
   389
blanchet@33197
   390
inductive_set S\<^isub>4 and A\<^isub>4 and B\<^isub>4 where
blanchet@33197
   391
  "[] \<in> S\<^isub>4"
blanchet@33197
   392
| "w \<in> A\<^isub>4 \<Longrightarrow> b # w \<in> S\<^isub>4"
blanchet@33197
   393
| "w \<in> B\<^isub>4 \<Longrightarrow> a # w \<in> S\<^isub>4"
blanchet@33197
   394
| "w \<in> S\<^isub>4 \<Longrightarrow> a # w \<in> A\<^isub>4"
blanchet@33197
   395
| "\<lbrakk>v \<in> A\<^isub>4; w \<in> A\<^isub>4\<rbrakk> \<Longrightarrow> b # v @ w \<in> A\<^isub>4"
blanchet@33197
   396
| "w \<in> S\<^isub>4 \<Longrightarrow> b # w \<in> B\<^isub>4"
blanchet@33197
   397
| "\<lbrakk>v \<in> B\<^isub>4; w \<in> B\<^isub>4\<rbrakk> \<Longrightarrow> a # v @ w \<in> B\<^isub>4"
blanchet@33197
   398
blanchet@33197
   399
theorem S\<^isub>4_sound:
blanchet@33197
   400
"w \<in> S\<^isub>4 \<longrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b]"
blanchet@35710
   401
nitpick [card = 1\<midarrow>6, expect = none]
blanchet@33197
   402
sorry
blanchet@33197
   403
blanchet@33197
   404
theorem S\<^isub>4_complete:
blanchet@33197
   405
"length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b] \<longrightarrow> w \<in> S\<^isub>4"
blanchet@35710
   406
nitpick [card = 1\<midarrow>6, expect = none]
blanchet@33197
   407
sorry
blanchet@33197
   408
blanchet@33197
   409
theorem S\<^isub>4_A\<^isub>4_B\<^isub>4_sound_and_complete:
blanchet@33197
   410
"w \<in> S\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b]"
blanchet@33197
   411
"w \<in> A\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b] + 1"
blanchet@33197
   412
"w \<in> B\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = b] = length [x \<leftarrow> w. x = a] + 1"
blanchet@35710
   413
nitpick [card = 1\<midarrow>6, expect = none]
blanchet@33197
   414
sorry
blanchet@33197
   415
blanchet@33197
   416
subsection {* 4.2. AA Trees *}
blanchet@33197
   417
blanchet@34969
   418
datatype 'a aa_tree = \<Lambda> | N "'a\<Colon>linorder" nat "'a aa_tree" "'a aa_tree"
blanchet@33197
   419
blanchet@33197
   420
primrec data where
blanchet@33197
   421
"data \<Lambda> = undefined" |
blanchet@33197
   422
"data (N x _ _ _) = x"
blanchet@33197
   423
blanchet@33197
   424
primrec dataset where
blanchet@33197
   425
"dataset \<Lambda> = {}" |
blanchet@33197
   426
"dataset (N x _ t u) = {x} \<union> dataset t \<union> dataset u"
blanchet@33197
   427
blanchet@33197
   428
primrec level where
blanchet@33197
   429
"level \<Lambda> = 0" |
blanchet@33197
   430
"level (N _ k _ _) = k"
blanchet@33197
   431
blanchet@33197
   432
primrec left where
blanchet@33197
   433
"left \<Lambda> = \<Lambda>" |
blanchet@33197
   434
"left (N _ _ t\<^isub>1 _) = t\<^isub>1"
blanchet@33197
   435
blanchet@33197
   436
primrec right where
blanchet@33197
   437
"right \<Lambda> = \<Lambda>" |
blanchet@33197
   438
"right (N _ _ _ t\<^isub>2) = t\<^isub>2"
blanchet@33197
   439
blanchet@33197
   440
fun wf where
blanchet@33197
   441
"wf \<Lambda> = True" |
blanchet@33197
   442
"wf (N _ k t u) =
blanchet@33197
   443
 (if t = \<Lambda> then
blanchet@33197
   444
    k = 1 \<and> (u = \<Lambda> \<or> (level u = 1 \<and> left u = \<Lambda> \<and> right u = \<Lambda>))
blanchet@33197
   445
  else
blanchet@33197
   446
    wf t \<and> wf u \<and> u \<noteq> \<Lambda> \<and> level t < k \<and> level u \<le> k \<and> level (right u) < k)"
blanchet@33197
   447
blanchet@33197
   448
fun skew where
blanchet@33197
   449
"skew \<Lambda> = \<Lambda>" |
blanchet@33197
   450
"skew (N x k t u) =
blanchet@33197
   451
 (if t \<noteq> \<Lambda> \<and> k = level t then
blanchet@33197
   452
    N (data t) k (left t) (N x k (right t) u)
blanchet@33197
   453
  else
blanchet@33197
   454
    N x k t u)"
blanchet@33197
   455
blanchet@33197
   456
fun split where
blanchet@33197
   457
"split \<Lambda> = \<Lambda>" |
blanchet@33197
   458
"split (N x k t u) =
blanchet@33197
   459
 (if u \<noteq> \<Lambda> \<and> k = level (right u) then
blanchet@33197
   460
    N (data u) (Suc k) (N x k t (left u)) (right u)
blanchet@33197
   461
  else
blanchet@33197
   462
    N x k t u)"
blanchet@33197
   463
blanchet@33197
   464
theorem dataset_skew_split:
blanchet@33197
   465
"dataset (skew t) = dataset t"
blanchet@33197
   466
"dataset (split t) = dataset t"
blanchet@35738
   467
nitpick [card = 1\<midarrow>5, expect = none]
blanchet@33197
   468
sorry
blanchet@33197
   469
blanchet@33197
   470
theorem wf_skew_split:
blanchet@33197
   471
"wf t \<Longrightarrow> skew t = t"
blanchet@33197
   472
"wf t \<Longrightarrow> split t = t"
blanchet@35738
   473
nitpick [card = 1\<midarrow>5, expect = none]
blanchet@33197
   474
sorry
blanchet@33197
   475
blanchet@33197
   476
primrec insort\<^isub>1 where
blanchet@33197
   477
"insort\<^isub>1 \<Lambda> x = N x 1 \<Lambda> \<Lambda>" |
blanchet@33197
   478
"insort\<^isub>1 (N y k t u) x =
blanchet@33197
   479
 (* (split \<circ> skew) *) (N y k (if x < y then insort\<^isub>1 t x else t)
blanchet@33197
   480
                             (if x > y then insort\<^isub>1 u x else u))"
blanchet@33197
   481
blanchet@33197
   482
theorem wf_insort\<^isub>1: "wf t \<Longrightarrow> wf (insort\<^isub>1 t x)"
blanchet@35666
   483
nitpick [expect = genuine]
blanchet@33197
   484
oops
blanchet@33197
   485
blanchet@33197
   486
theorem wf_insort\<^isub>1_nat: "wf t \<Longrightarrow> wf (insort\<^isub>1 t (x\<Colon>nat))"
blanchet@35666
   487
nitpick [eval = "insort\<^isub>1 t x", expect = genuine]
blanchet@33197
   488
oops
blanchet@33197
   489
blanchet@33197
   490
primrec insort\<^isub>2 where
blanchet@33197
   491
"insort\<^isub>2 \<Lambda> x = N x 1 \<Lambda> \<Lambda>" |
blanchet@33197
   492
"insort\<^isub>2 (N y k t u) x =
blanchet@33197
   493
 (split \<circ> skew) (N y k (if x < y then insort\<^isub>2 t x else t)
blanchet@33197
   494
                       (if x > y then insort\<^isub>2 u x else u))"
blanchet@33197
   495
blanchet@33197
   496
theorem wf_insort\<^isub>2: "wf t \<Longrightarrow> wf (insort\<^isub>2 t x)"
blanchet@35738
   497
nitpick [card = 1\<midarrow>5, expect = none]
blanchet@33197
   498
sorry
blanchet@33197
   499
blanchet@33197
   500
theorem dataset_insort\<^isub>2: "dataset (insort\<^isub>2 t x) = {x} \<union> dataset t"
blanchet@35738
   501
nitpick [card = 1\<midarrow>5, expect = none]
blanchet@33197
   502
sorry
blanchet@33197
   503
blanchet@33197
   504
end