src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy
author wenzelm
Tue, 19 Dec 2017 13:58:12 +0100
changeset 67226 ec32cdaab97b
parent 66453 cc19f7ca2ed6
child 67399 eab6ce8368fa
permissions -rw-r--r--
isabelle update_cartouches -c -t;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
     1
theory Predicate_Compile_Tests
66453
cc19f7ca2ed6 session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents: 66283
diff changeset
     2
imports "HOL-Library.Predicate_Compile_Alternative_Defs"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
     3
begin
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
     4
42208
02513eb26eb7 raised timeouts further, for SML/NJ -- because of variations in machines/compilers, fixed timeouts can merely prevent non-termination, not enforce particular performance characteristics.
krauss
parents: 42142
diff changeset
     5
declare [[values_timeout = 480.0]]
42142
d24a93025feb raised various timeouts to accommodate sluggish SML/NJ
krauss
parents: 41413
diff changeset
     6
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
     7
subsection \<open>Basic predicates\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
     8
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
     9
inductive False' :: "bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    10
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    11
code_pred (expected_modes: bool) False' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    12
code_pred [dseq] False' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    13
code_pred [random_dseq] False' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    14
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    15
values [expected "{}" pred] "{x. False'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    16
values [expected "{}" dseq 1] "{x. False'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    17
values [expected "{}" random_dseq 1, 1, 1] "{x. False'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    18
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    19
value "False'"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    20
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    21
inductive True' :: "bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    22
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    23
  "True ==> True'"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    24
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    25
code_pred True' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    26
code_pred [dseq] True' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    27
code_pred [random_dseq] True' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    28
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    29
thm True'.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    30
thm True'.dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    31
thm True'.random_dseq_equation
51143
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
    32
values [expected "{()}"] "{x. True'}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    33
values [expected "{}" dseq 0] "{x. True'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    34
values [expected "{()}" dseq 1] "{x. True'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    35
values [expected "{()}" dseq 2] "{x. True'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    36
values [expected "{}" random_dseq 1, 1, 0] "{x. True'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    37
values [expected "{}" random_dseq 1, 1, 1] "{x. True'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    38
values [expected "{()}" random_dseq 1, 1, 2] "{x. True'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    39
values [expected "{()}" random_dseq 1, 1, 3] "{x. True'}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    40
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
    41
inductive EmptyPred :: "'a \<Rightarrow> bool"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    42
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
    43
code_pred (expected_modes: o => bool, i => bool) EmptyPred .
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    44
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
    45
definition EmptyPred' :: "'a \<Rightarrow> bool"
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
    46
where "EmptyPred' = (\<lambda> x. False)"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    47
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
    48
code_pred (expected_modes: o => bool, i => bool) [inductify] EmptyPred' .
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    49
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    50
inductive EmptyRel :: "'a \<Rightarrow> 'b \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    51
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    52
code_pred (expected_modes: o => o => bool, i => o => bool, o => i => bool, i => i => bool) EmptyRel .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    53
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    54
inductive EmptyClosure :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    55
for r :: "'a \<Rightarrow> 'a \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    56
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    57
code_pred
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    58
  (expected_modes: (o => o => bool) => o => o => bool, (o => o => bool) => i => o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    59
         (o => o => bool) => o => i => bool, (o => o => bool) => i => i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    60
         (i => o => bool) => o => o => bool, (i => o => bool) => i => o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    61
         (i => o => bool) => o => i => bool, (i => o => bool) => i => i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    62
         (o => i => bool) => o => o => bool, (o => i => bool) => i => o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    63
         (o => i => bool) => o => i => bool, (o => i => bool) => i => i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    64
         (i => i => bool) => o => o => bool, (i => i => bool) => i => o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    65
         (i => i => bool) => o => i => bool, (i => i => bool) => i => i => bool)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    66
  EmptyClosure .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    67
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    68
thm EmptyClosure.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    69
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    70
(* TODO: inductive package is broken!
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    71
inductive False'' :: "bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    72
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    73
  "False \<Longrightarrow> False''"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    74
40100
98d74bbe8cd8 updating to new notation in commented examples
bulwahn
parents: 39803
diff changeset
    75
code_pred (expected_modes: bool) False'' .
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    76
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    77
inductive EmptySet'' :: "'a \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    78
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    79
  "False \<Longrightarrow> EmptySet'' x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    80
40100
98d74bbe8cd8 updating to new notation in commented examples
bulwahn
parents: 39803
diff changeset
    81
code_pred (expected_modes: i => bool, o => bool) [inductify] EmptySet'' .
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    82
*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    83
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    84
consts a' :: 'a
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    85
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    86
inductive Fact :: "'a \<Rightarrow> 'a \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    87
where
62121
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
    88
  "Fact a' a'"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    89
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    90
code_pred (expected_modes: o => o => bool, i => o => bool, o => i => bool, i => i => bool) Fact .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
    91
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
    92
text \<open>
62121
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
    93
  The following example was derived from an predicate in the CakeML formalisation provided by Lars Hupel.
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
    94
\<close>
62121
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
    95
inductive predicate_where_argument_is_condition :: "bool \<Rightarrow> bool"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
    96
where
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
    97
  "ck \<Longrightarrow> predicate_where_argument_is_condition ck"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
    98
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
    99
code_pred predicate_where_argument_is_condition .
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   100
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   101
text \<open>Other similar examples of this kind:\<close>
62121
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   102
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   103
inductive predicate_where_argument_is_in_equation :: "bool \<Rightarrow> bool"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   104
where
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   105
  "ck = True \<Longrightarrow> predicate_where_argument_is_in_equation ck"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   106
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   107
code_pred predicate_where_argument_is_in_equation .
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   108
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   109
inductive predicate_where_argument_is_condition_and_value :: "bool \<Rightarrow> bool"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   110
where
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   111
  "predicate_where_argument_is_condition_and_value ck \<Longrightarrow> ck
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   112
     \<Longrightarrow> predicate_where_argument_is_condition_and_value ck"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   113
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   114
code_pred predicate_where_argument_is_condition_and_value .
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   115
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   116
inductive predicate_where_argument_is_neg_condition :: "bool \<Rightarrow> bool"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   117
where
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   118
  "\<not> ck \<Longrightarrow> predicate_where_argument_is_neg_condition ck"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   119
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   120
code_pred predicate_where_argument_is_neg_condition .
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   121
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   122
inductive predicate_where_argument_is_neg_condition_and_in_equation :: "bool \<Rightarrow> bool"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   123
where
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   124
  "\<not> ck \<Longrightarrow> ck = False \<Longrightarrow> predicate_where_argument_is_neg_condition_and_in_equation ck"
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   125
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   126
code_pred predicate_where_argument_is_neg_condition_and_in_equation .
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   127
67226
ec32cdaab97b isabelle update_cartouches -c -t;
wenzelm
parents: 66453
diff changeset
   128
text \<open>Another related example that required slight adjustment of the proof procedure\<close>
64542
c7d76708379f filter non-matching prems to not fail in proof procedure; include test case (related to c8a93680b80d)
bulwahn
parents: 63167
diff changeset
   129
c7d76708379f filter non-matching prems to not fail in proof procedure; include test case (related to c8a93680b80d)
bulwahn
parents: 63167
diff changeset
   130
inductive if_as_predicate :: "bool \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"
c7d76708379f filter non-matching prems to not fail in proof procedure; include test case (related to c8a93680b80d)
bulwahn
parents: 63167
diff changeset
   131
where
c7d76708379f filter non-matching prems to not fail in proof procedure; include test case (related to c8a93680b80d)
bulwahn
parents: 63167
diff changeset
   132
  "condition \<Longrightarrow> if_as_predicate condition then_value else_value then_value"
c7d76708379f filter non-matching prems to not fail in proof procedure; include test case (related to c8a93680b80d)
bulwahn
parents: 63167
diff changeset
   133
| "\<not> condition \<Longrightarrow> if_as_predicate condition then_value else_value else_value"
c7d76708379f filter non-matching prems to not fail in proof procedure; include test case (related to c8a93680b80d)
bulwahn
parents: 63167
diff changeset
   134
c7d76708379f filter non-matching prems to not fail in proof procedure; include test case (related to c8a93680b80d)
bulwahn
parents: 63167
diff changeset
   135
code_pred [show_proof_trace] if_as_predicate .
62121
c8a93680b80d filter non-matching prems rather than fail in proof procedure in rare cases; include derived example motivating change and some similar other ones
Lukas Bulwahn <lukas.bulwahn@gmail.com>
parents: 60565
diff changeset
   136
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   137
inductive zerozero :: "nat * nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   138
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   139
  "zerozero (0, 0)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   140
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   141
code_pred (expected_modes: i => bool, i * o => bool, o * i => bool, o => bool) zerozero .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   142
code_pred [dseq] zerozero .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   143
code_pred [random_dseq] zerozero .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   144
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   145
thm zerozero.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   146
thm zerozero.dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   147
thm zerozero.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   148
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   149
text \<open>We expect the user to expand the tuples in the values command.
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   150
The following values command is not supported.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   151
(*values "{x. zerozero x}" *)
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   152
text \<open>Instead, the user must type\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   153
values "{(x, y). zerozero (x, y)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   154
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   155
values [expected "{}" dseq 0] "{(x, y). zerozero (x, y)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   156
values [expected "{(0::nat, 0::nat)}" dseq 1] "{(x, y). zerozero (x, y)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   157
values [expected "{(0::nat, 0::nat)}" dseq 2] "{(x, y). zerozero (x, y)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   158
values [expected "{}" random_dseq 1, 1, 2] "{(x, y). zerozero (x, y)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   159
values [expected "{(0::nat, 0:: nat)}" random_dseq 1, 1, 3] "{(x, y). zerozero (x, y)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   160
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   161
inductive nested_tuples :: "((int * int) * int * int) => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   162
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   163
  "nested_tuples ((0, 1), 2, 3)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   164
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   165
code_pred nested_tuples .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   166
51143
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   167
inductive JamesBond :: "nat => int => natural => bool"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   168
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   169
  "JamesBond 0 0 7"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   170
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   171
code_pred JamesBond .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   172
51143
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   173
values [expected "{(0::nat, 0::int , 7::natural)}"] "{(a, b, c). JamesBond a b c}"
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   174
values [expected "{(0::nat, 7::natural, 0:: int)}"] "{(a, c, b). JamesBond a b c}"
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   175
values [expected "{(0::int, 0::nat, 7::natural)}"] "{(b, a, c). JamesBond a b c}"
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   176
values [expected "{(0::int, 7::natural, 0::nat)}"] "{(b, c, a). JamesBond a b c}"
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   177
values [expected "{(7::natural, 0::nat, 0::int)}"] "{(c, a, b). JamesBond a b c}"
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   178
values [expected "{(7::natural, 0::int, 0::nat)}"] "{(c, b, a). JamesBond a b c}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   179
51143
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   180
values [expected "{(7::natural, 0::int)}"] "{(a, b). JamesBond 0 b a}"
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   181
values [expected "{(7::natural, 0::nat)}"] "{(c, a). JamesBond a 0 c}"
0a2371e7ced3 two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents: 47433
diff changeset
   182
values [expected "{(0::nat, 7::natural)}"] "{(a, c). JamesBond a 0 c}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   183
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   184
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   185
subsection \<open>Alternative Rules\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   186
58310
91ea607a34d8 updated news
blanchet
parents: 58249
diff changeset
   187
datatype char = C | D | E | F | G | H
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   188
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   189
inductive is_C_or_D
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   190
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   191
  "(x = C) \<or> (x = D) ==> is_C_or_D x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   192
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   193
code_pred (expected_modes: i => bool) is_C_or_D .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   194
thm is_C_or_D.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   195
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   196
inductive is_D_or_E
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   197
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   198
  "(x = D) \<or> (x = E) ==> is_D_or_E x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   199
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   200
lemma [code_pred_intro]:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   201
  "is_D_or_E D"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   202
by (auto intro: is_D_or_E.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   203
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   204
lemma [code_pred_intro]:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   205
  "is_D_or_E E"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   206
by (auto intro: is_D_or_E.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   207
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   208
code_pred (expected_modes: o => bool, i => bool) is_D_or_E
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   209
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   210
  case is_D_or_E
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   211
  from is_D_or_E.prems show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   212
  proof 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   213
    fix xa
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   214
    assume x: "x = xa"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   215
    assume "xa = D \<or> xa = E"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   216
    from this show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   217
    proof
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   218
      assume "xa = D" from this x is_D_or_E(1) show thesis by simp
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   219
    next
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   220
      assume "xa = E" from this x is_D_or_E(2) show thesis by simp
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   221
    qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   222
  qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   223
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   224
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   225
thm is_D_or_E.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   226
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   227
inductive is_F_or_G
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   228
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   229
  "x = F \<or> x = G ==> is_F_or_G x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   230
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   231
lemma [code_pred_intro]:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   232
  "is_F_or_G F"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   233
by (auto intro: is_F_or_G.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   234
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   235
lemma [code_pred_intro]:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   236
  "is_F_or_G G"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   237
by (auto intro: is_F_or_G.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   238
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   239
inductive is_FGH
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   240
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   241
  "is_F_or_G x ==> is_FGH x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   242
| "is_FGH H"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   243
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   244
text \<open>Compilation of is_FGH requires elimination rule for is_F_or_G\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   245
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   246
code_pred (expected_modes: o => bool, i => bool) is_FGH
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   247
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   248
  case is_F_or_G
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   249
  from is_F_or_G.prems show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   250
  proof
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   251
    fix xa
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   252
    assume x: "x = xa"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   253
    assume "xa = F \<or> xa = G"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   254
    from this show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   255
    proof
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   256
      assume "xa = F"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   257
      from this x is_F_or_G(1) show thesis by simp
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   258
    next
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   259
      assume "xa = G"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   260
      from this x is_F_or_G(2) show thesis by simp
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   261
    qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   262
  qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   263
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   264
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   265
subsection \<open>Named alternative rules\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   266
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   267
inductive appending
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   268
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   269
  nil: "appending [] ys ys"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   270
| cons: "appending xs ys zs \<Longrightarrow> appending (x#xs) ys (x#zs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   271
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   272
lemma appending_alt_nil: "ys = zs \<Longrightarrow> appending [] ys zs"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   273
by (auto intro: appending.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   274
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   275
lemma appending_alt_cons: "xs' = x # xs \<Longrightarrow> appending xs ys zs \<Longrightarrow> zs' = x # zs \<Longrightarrow> appending xs' ys zs'"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   276
by (auto intro: appending.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   277
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   278
text \<open>With code_pred_intro, we can give fact names to the alternative rules,
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   279
  which are used for the code_pred command.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   280
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   281
declare appending_alt_nil[code_pred_intro alt_nil] appending_alt_cons[code_pred_intro alt_cons]
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   282
 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   283
code_pred appending
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   284
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   285
  case appending
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   286
  from appending.prems show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   287
  proof(cases)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   288
    case nil
60565
b7ee41f72add clarified 'case' command;
wenzelm
parents: 58310
diff changeset
   289
    from appending.alt_nil nil show thesis by auto
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   290
  next
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   291
    case cons
60565
b7ee41f72add clarified 'case' command;
wenzelm
parents: 58310
diff changeset
   292
    from appending.alt_cons cons show thesis by fastforce
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   293
  qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   294
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   295
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   296
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   297
inductive ya_even and ya_odd :: "nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   298
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   299
  even_zero: "ya_even 0"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   300
| odd_plus1: "ya_even x ==> ya_odd (x + 1)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   301
| even_plus1: "ya_odd x ==> ya_even (x + 1)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   302
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   303
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   304
declare even_zero[code_pred_intro even_0]
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   305
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   306
lemma [code_pred_intro odd_Suc]: "ya_even x ==> ya_odd (Suc x)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   307
by (auto simp only: Suc_eq_plus1 intro: ya_even_ya_odd.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   308
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   309
lemma [code_pred_intro even_Suc]:"ya_odd x ==> ya_even (Suc x)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   310
by (auto simp only: Suc_eq_plus1 intro: ya_even_ya_odd.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   311
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   312
code_pred ya_even
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   313
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   314
  case ya_even
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   315
  from ya_even.prems show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   316
  proof (cases)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   317
    case even_zero
60565
b7ee41f72add clarified 'case' command;
wenzelm
parents: 58310
diff changeset
   318
    from even_zero ya_even.even_0 show thesis by simp
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   319
  next
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   320
    case even_plus1
60565
b7ee41f72add clarified 'case' command;
wenzelm
parents: 58310
diff changeset
   321
    from even_plus1 ya_even.even_Suc show thesis by simp
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   322
  qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   323
next
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   324
  case ya_odd
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   325
  from ya_odd.prems show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   326
  proof (cases)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   327
    case odd_plus1
60565
b7ee41f72add clarified 'case' command;
wenzelm
parents: 58310
diff changeset
   328
    from odd_plus1 ya_odd.odd_Suc show thesis by simp
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   329
  qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   330
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   331
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   332
subsection \<open>Preprocessor Inlining\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   333
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   334
definition "equals == (op =)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   335
 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   336
inductive zerozero' :: "nat * nat => bool" where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   337
  "equals (x, y) (0, 0) ==> zerozero' (x, y)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   338
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   339
code_pred (expected_modes: i => bool) zerozero' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   340
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   341
lemma zerozero'_eq: "zerozero' x == zerozero x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   342
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   343
  have "zerozero' = zerozero"
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   344
    apply (auto simp add: fun_eq_iff)
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   345
    apply (cases rule: zerozero'.cases)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   346
    apply (auto simp add: equals_def intro: zerozero.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   347
    apply (cases rule: zerozero.cases)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   348
    apply (auto simp add: equals_def intro: zerozero'.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   349
    done
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   350
  from this show "zerozero' x == zerozero x" by auto
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   351
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   352
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   353
declare zerozero'_eq [code_pred_inline]
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   354
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   355
definition "zerozero'' x == zerozero' x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   356
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   357
text \<open>if preprocessing fails, zerozero'' will not have all modes.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   358
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   359
code_pred (expected_modes: i * i => bool, i * o => bool, o * i => bool, o => bool) [inductify] zerozero'' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   360
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   361
subsection \<open>Sets\<close>
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   362
(*
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   363
inductive_set EmptySet :: "'a set"
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   364
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   365
code_pred (expected_modes: o => bool, i => bool) EmptySet .
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   366
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   367
definition EmptySet' :: "'a set"
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   368
where "EmptySet' = {}"
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   369
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   370
code_pred (expected_modes: o => bool, i => bool) [inductify] EmptySet' .
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   371
*)
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   372
subsection \<open>Numerals\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   373
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   374
definition
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   375
  "one_or_two = (%x. x = Suc 0 \<or> ( x = Suc (Suc 0)))"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   376
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   377
code_pred [inductify] one_or_two .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   378
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   379
code_pred [dseq] one_or_two .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   380
code_pred [random_dseq] one_or_two .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   381
thm one_or_two.dseq_equation
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
   382
values [expected "{1::nat, 2}"] "{x. one_or_two x}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   383
values [random_dseq 0,0,10] 3 "{x. one_or_two x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   384
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   385
inductive one_or_two' :: "nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   386
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   387
  "one_or_two' 1"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   388
| "one_or_two' 2"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   389
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   390
code_pred one_or_two' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   391
thm one_or_two'.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   392
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   393
values "{x. one_or_two' x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   394
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   395
definition one_or_two'':
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   396
  "one_or_two'' == (%x. x = 1 \<or> x = (2::nat))"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   397
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   398
code_pred [inductify] one_or_two'' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   399
thm one_or_two''.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   400
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   401
values "{x. one_or_two'' x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   402
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   403
subsection \<open>even predicate\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   404
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   405
inductive even :: "nat \<Rightarrow> bool" and odd :: "nat \<Rightarrow> bool" where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   406
    "even 0"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   407
  | "even n \<Longrightarrow> odd (Suc n)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   408
  | "odd n \<Longrightarrow> even (Suc n)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   409
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   410
code_pred (expected_modes: i => bool, o => bool) even .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   411
code_pred [dseq] even .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   412
code_pred [random_dseq] even .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   413
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   414
thm odd.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   415
thm even.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   416
thm odd.dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   417
thm even.dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   418
thm odd.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   419
thm even.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   420
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   421
values "{x. even 2}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   422
values "{x. odd 2}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   423
values 10 "{n. even n}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   424
values 10 "{n. odd n}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   425
values [expected "{}" dseq 2] "{x. even 6}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   426
values [expected "{}" dseq 6] "{x. even 6}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   427
values [expected "{()}" dseq 7] "{x. even 6}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   428
values [dseq 2] "{x. odd 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   429
values [dseq 6] "{x. odd 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   430
values [dseq 7] "{x. odd 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   431
values [expected "{()}" dseq 8] "{x. odd 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   432
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   433
values [expected "{}" dseq 0] 8 "{x. even x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   434
values [expected "{0::nat}" dseq 1] 8 "{x. even x}"
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
   435
values [expected "{0::nat, 2}" dseq 3] 8 "{x. even x}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
   436
values [expected "{0::nat, 2}" dseq 4] 8 "{x. even x}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
   437
values [expected "{0::nat, 2, 4}" dseq 6] 8 "{x. even x}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   438
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   439
values [random_dseq 1, 1, 0] 8 "{x. even x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   440
values [random_dseq 1, 1, 1] 8 "{x. even x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   441
values [random_dseq 1, 1, 2] 8 "{x. even x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   442
values [random_dseq 1, 1, 3] 8 "{x. even x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   443
values [random_dseq 1, 1, 6] 8 "{x. even x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   444
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   445
values [expected "{}" random_dseq 1, 1, 7] "{x. odd 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   446
values [random_dseq 1, 1, 8] "{x. odd 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   447
values [random_dseq 1, 1, 9] "{x. odd 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   448
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   449
definition odd' where "odd' x == \<not> even x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   450
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   451
code_pred (expected_modes: i => bool) [inductify] odd' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   452
code_pred [dseq inductify] odd' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   453
code_pred [random_dseq inductify] odd' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   454
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   455
values [expected "{}" dseq 2] "{x. odd' 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   456
values [expected "{()}" dseq 9] "{x. odd' 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   457
values [expected "{}" dseq 2] "{x. odd' 8}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   458
values [expected "{}" dseq 10] "{x. odd' 8}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   459
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   460
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   461
inductive is_even :: "nat \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   462
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   463
  "n mod 2 = 0 \<Longrightarrow> is_even n"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   464
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   465
code_pred (expected_modes: i => bool) is_even .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   466
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   467
subsection \<open>append predicate\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   468
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   469
inductive append :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list \<Rightarrow> bool" where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   470
    "append [] xs xs"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   471
  | "append xs ys zs \<Longrightarrow> append (x # xs) ys (x # zs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   472
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   473
code_pred (modes: i => i => o => bool as "concat", o => o => i => bool as "slice", o => i => i => bool as prefix,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   474
  i => o => i => bool as suffix, i => i => i => bool) append .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   475
code_pred (modes: i \<Rightarrow> i \<Rightarrow> o \<Rightarrow> bool as "concat", o \<Rightarrow> o \<Rightarrow> i \<Rightarrow> bool as "slice", o \<Rightarrow> i \<Rightarrow> i \<Rightarrow> bool as prefix,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   476
  i \<Rightarrow> o \<Rightarrow> i \<Rightarrow> bool as suffix, i \<Rightarrow> i \<Rightarrow> i \<Rightarrow> bool) append .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   477
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   478
code_pred [dseq] append .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   479
code_pred [random_dseq] append .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   480
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   481
thm append.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   482
thm append.dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   483
thm append.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   484
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   485
values "{(ys, xs). append xs ys [0, Suc 0, 2]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   486
values "{zs. append [0, Suc 0, 2] [17, 8] zs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   487
values "{ys. append [0, Suc 0, 2] ys [0, Suc 0, 2, 17, 0, 5]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   488
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   489
values [expected "{}" dseq 0] 10 "{(xs, ys). append xs ys [1, 2, 3, 4, (5::nat)]}"
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
   490
values [expected "{(([]::nat list), [1::nat, 2, 3, 4, 5])}" dseq 1] 10 "{(xs, ys). append xs ys [1, 2, 3, 4, (5::nat)]}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   491
values [dseq 4] 10 "{(xs, ys). append xs ys [1, 2, 3, 4, (5::nat)]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   492
values [dseq 6] 10 "{(xs, ys). append xs ys [1, 2, 3, 4, (5::nat)]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   493
values [random_dseq 1, 1, 4] 10 "{(xs, ys). append xs ys [1, 2, 3, 4, (5::nat)]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   494
values [random_dseq 1, 1, 1] 10 "{(xs, ys, zs::int list). append xs ys zs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   495
values [random_dseq 1, 1, 3] 10 "{(xs, ys, zs::int list). append xs ys zs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   496
values [random_dseq 3, 1, 3] 10 "{(xs, ys, zs::int list). append xs ys zs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   497
values [random_dseq 1, 3, 3] 10 "{(xs, ys, zs::int list). append xs ys zs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   498
values [random_dseq 1, 1, 4] 10 "{(xs, ys, zs::int list). append xs ys zs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   499
56927
4044a7d1720f hardcoded nbe and sml into value command
haftmann
parents: 56679
diff changeset
   500
value "Predicate.the (concat [0::int, 1, 2] [3, 4, 5])"
4044a7d1720f hardcoded nbe and sml into value command
haftmann
parents: 56679
diff changeset
   501
value "Predicate.the (slice ([]::int list))"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   502
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   503
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   504
text \<open>tricky case with alternative rules\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   505
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   506
inductive append2
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   507
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   508
  "append2 [] xs xs"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   509
| "append2 xs ys zs \<Longrightarrow> append2 (x # xs) ys (x # zs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   510
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   511
lemma append2_Nil: "append2 [] (xs::'b list) xs"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   512
  by (simp add: append2.intros(1))
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   513
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   514
lemmas [code_pred_intro] = append2_Nil append2.intros(2)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   515
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   516
code_pred (expected_modes: i => i => o => bool, o => o => i => bool, o => i => i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   517
  i => o => i => bool, i => i => i => bool) append2
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   518
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   519
  case append2
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   520
  from append2.prems show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   521
  proof
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   522
    fix xs
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   523
    assume "xa = []" "xb = xs" "xc = xs"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   524
    from this append2(1) show thesis by simp
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   525
  next
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   526
    fix xs ys zs x
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   527
    assume "xa = x # xs" "xb = ys" "xc = x # zs" "append2 xs ys zs"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42463
diff changeset
   528
    from this append2(2) show thesis by fastforce
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   529
  qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   530
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   531
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   532
inductive tupled_append :: "'a list \<times> 'a list \<times> 'a list \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   533
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   534
  "tupled_append ([], xs, xs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   535
| "tupled_append (xs, ys, zs) \<Longrightarrow> tupled_append (x # xs, ys, x # zs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   536
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   537
code_pred (expected_modes: i * i * o => bool, o * o * i => bool, o * i * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   538
  i * o * i => bool, i * i * i => bool) tupled_append .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   539
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   540
code_pred (expected_modes: i \<times> i \<times> o \<Rightarrow> bool, o \<times> o \<times> i \<Rightarrow> bool, o \<times> i \<times> i \<Rightarrow> bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   541
  i \<times> o \<times> i \<Rightarrow> bool, i \<times> i \<times> i \<Rightarrow> bool) tupled_append .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   542
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   543
code_pred [random_dseq] tupled_append .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   544
thm tupled_append.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   545
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   546
values "{xs. tupled_append ([(1::nat), 2, 3], [4, 5], xs)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   547
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   548
inductive tupled_append'
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   549
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   550
"tupled_append' ([], xs, xs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   551
| "[| ys = fst (xa, y); x # zs = snd (xa, y);
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   552
 tupled_append' (xs, ys, zs) |] ==> tupled_append' (x # xs, xa, y)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   553
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   554
code_pred (expected_modes: i * i * o => bool, o * o * i => bool, o * i * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   555
  i * o * i => bool, i * i * i => bool) tupled_append' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   556
thm tupled_append'.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   557
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   558
inductive tupled_append'' :: "'a list \<times> 'a list \<times> 'a list \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   559
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   560
  "tupled_append'' ([], xs, xs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   561
| "ys = fst yszs ==> x # zs = snd yszs ==> tupled_append'' (xs, ys, zs) \<Longrightarrow> tupled_append'' (x # xs, yszs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   562
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   563
code_pred (expected_modes: i * i * o => bool, o * o * i => bool, o * i * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   564
  i * o * i => bool, i * i * i => bool) tupled_append'' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   565
thm tupled_append''.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   566
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   567
inductive tupled_append''' :: "'a list \<times> 'a list \<times> 'a list \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   568
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   569
  "tupled_append''' ([], xs, xs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   570
| "yszs = (ys, zs) ==> tupled_append''' (xs, yszs) \<Longrightarrow> tupled_append''' (x # xs, ys, x # zs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   571
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   572
code_pred (expected_modes: i * i * o => bool, o * o * i => bool, o * i * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   573
  i * o * i => bool, i * i * i => bool) tupled_append''' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   574
thm tupled_append'''.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   575
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   576
subsection \<open>map_ofP predicate\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   577
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   578
inductive map_ofP :: "('a \<times> 'b) list \<Rightarrow> 'a \<Rightarrow> 'b \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   579
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   580
  "map_ofP ((a, b)#xs) a b"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   581
| "map_ofP xs a b \<Longrightarrow> map_ofP (x#xs) a b"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   582
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   583
code_pred (expected_modes: i => o => o => bool, i => i => o => bool, i => o => i => bool, i => i => i => bool) map_ofP .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   584
thm map_ofP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   585
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   586
subsection \<open>filter predicate\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   587
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   588
inductive filter1
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   589
for P
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   590
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   591
  "filter1 P [] []"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   592
| "P x ==> filter1 P xs ys ==> filter1 P (x#xs) (x#ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   593
| "\<not> P x ==> filter1 P xs ys ==> filter1 P (x#xs) ys"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   594
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   595
code_pred (expected_modes: (i => bool) => i => o => bool, (i => bool) => i => i => bool) filter1 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   596
code_pred [dseq] filter1 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   597
code_pred [random_dseq] filter1 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   598
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   599
thm filter1.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   600
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
   601
values [expected "{[0::nat, 2, 4]}"] "{xs. filter1 even [0, 1, 2, 3, 4] xs}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   602
values [expected "{}" dseq 9] "{xs. filter1 even [0, 1, 2, 3, 4] xs}"
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
   603
values [expected "{[0::nat, 2, 4]}" dseq 10] "{xs. filter1 even [0, 1, 2, 3, 4] xs}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   604
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   605
inductive filter2
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   606
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   607
  "filter2 P [] []"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   608
| "P x ==> filter2 P xs ys ==> filter2 P (x#xs) (x#ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   609
| "\<not> P x ==> filter2 P xs ys ==> filter2 P (x#xs) ys"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   610
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   611
code_pred (expected_modes: (i => bool) => i => i => bool, (i => bool) => i => o => bool) filter2 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   612
code_pred [dseq] filter2 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   613
code_pred [random_dseq] filter2 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   614
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   615
thm filter2.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   616
thm filter2.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   617
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   618
inductive filter3
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   619
for P
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   620
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   621
  "List.filter P xs = ys ==> filter3 P xs ys"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   622
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   623
code_pred (expected_modes: (o => bool) => i => o => bool, (o => bool) => i => i => bool , (i => bool) => i => o => bool, (i => bool) => i => i => bool) [skip_proof] filter3 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   624
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   625
code_pred filter3 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   626
thm filter3.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   627
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   628
(*
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   629
inductive filter4
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   630
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   631
  "List.filter P xs = ys ==> filter4 P xs ys"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   632
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   633
code_pred (expected_modes: i => i => o => bool, i => i => i => bool) filter4 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   634
(*code_pred [depth_limited] filter4 .*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   635
(*code_pred [random] filter4 .*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   636
*)
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   637
subsection \<open>reverse predicate\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   638
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   639
inductive rev where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   640
    "rev [] []"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   641
  | "rev xs xs' ==> append xs' [x] ys ==> rev (x#xs) ys"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   642
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   643
code_pred (expected_modes: i => o => bool, o => i => bool, i => i => bool) rev .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   644
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   645
thm rev.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   646
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   647
values "{xs. rev [0, 1, 2, 3::nat] xs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   648
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   649
inductive tupled_rev where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   650
  "tupled_rev ([], [])"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   651
| "tupled_rev (xs, xs') \<Longrightarrow> tupled_append (xs', [x], ys) \<Longrightarrow> tupled_rev (x#xs, ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   652
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   653
code_pred (expected_modes: i * o => bool, o * i => bool, i * i => bool) tupled_rev .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   654
thm tupled_rev.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   655
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   656
subsection \<open>partition predicate\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   657
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   658
inductive partition :: "('a \<Rightarrow> bool) \<Rightarrow> 'a list \<Rightarrow> 'a list \<Rightarrow> 'a list \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   659
  for f where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   660
    "partition f [] [] []"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   661
  | "f x \<Longrightarrow> partition f xs ys zs \<Longrightarrow> partition f (x # xs) (x # ys) zs"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   662
  | "\<not> f x \<Longrightarrow> partition f xs ys zs \<Longrightarrow> partition f (x # xs) ys (x # zs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   663
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   664
code_pred (expected_modes: (i => bool) => i => o => o => bool, (i => bool) => o => i => i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   665
  (i => bool) => i => i => o => bool, (i => bool) => i => o => i => bool, (i => bool) => i => i => i => bool)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   666
  partition .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   667
code_pred [dseq] partition .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   668
code_pred [random_dseq] partition .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   669
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   670
values 10 "{(ys, zs). partition is_even
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   671
  [0, Suc 0, 2, 3, 4, 5, 6, 7] ys zs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   672
values 10 "{zs. partition is_even zs [0, 2] [3, 5]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   673
values 10 "{zs. partition is_even zs [0, 7] [3, 5]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   674
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   675
inductive tupled_partition :: "('a \<Rightarrow> bool) \<Rightarrow> ('a list \<times> 'a list \<times> 'a list) \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   676
  for f where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   677
   "tupled_partition f ([], [], [])"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   678
  | "f x \<Longrightarrow> tupled_partition f (xs, ys, zs) \<Longrightarrow> tupled_partition f (x # xs, x # ys, zs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   679
  | "\<not> f x \<Longrightarrow> tupled_partition f (xs, ys, zs) \<Longrightarrow> tupled_partition f (x # xs, ys, x # zs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   680
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   681
code_pred (expected_modes: (i => bool) => i => bool, (i => bool) => (i * i * o) => bool, (i => bool) => (i * o * i) => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   682
  (i => bool) => (o * i * i) => bool, (i => bool) => (i * o * o) => bool) tupled_partition .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   683
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   684
thm tupled_partition.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   685
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   686
lemma [code_pred_intro]:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   687
  "r a b \<Longrightarrow> tranclp r a b"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   688
  "r a b \<Longrightarrow> tranclp r b c \<Longrightarrow> tranclp r a c"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   689
  by auto
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   690
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   691
subsection \<open>transitive predicate\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   692
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   693
text \<open>Also look at the tabled transitive closure in the Library\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   694
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   695
code_pred (modes: (i => o => bool) => i => i => bool, (i => o => bool) => i => o => bool as forwards_trancl,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   696
  (o => i => bool) => i => i => bool, (o => i => bool) => o => i => bool as backwards_trancl, (o => o => bool) => i => i => bool, (o => o => bool) => i => o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   697
  (o => o => bool) => o => i => bool, (o => o => bool) => o => o => bool) tranclp
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   698
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   699
  case tranclp
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   700
  from this converse_tranclpE[OF tranclp.prems] show thesis by metis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   701
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   702
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   703
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   704
code_pred [dseq] tranclp .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   705
code_pred [random_dseq] tranclp .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   706
thm tranclp.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   707
thm tranclp.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   708
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   709
inductive rtrancl' :: "'a => 'a => ('a => 'a => bool) => bool" 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   710
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   711
  "rtrancl' x x r"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   712
| "r x y ==> rtrancl' y z r ==> rtrancl' x z r"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   713
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   714
code_pred [random_dseq] rtrancl' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   715
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   716
thm rtrancl'.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   717
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   718
inductive rtrancl'' :: "('a * 'a * ('a \<Rightarrow> 'a \<Rightarrow> bool)) \<Rightarrow> bool"  
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   719
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   720
  "rtrancl'' (x, x, r)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   721
| "r x y \<Longrightarrow> rtrancl'' (y, z, r) \<Longrightarrow> rtrancl'' (x, z, r)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   722
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   723
code_pred rtrancl'' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   724
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   725
inductive rtrancl''' :: "('a * ('a * 'a) * ('a * 'a => bool)) => bool" 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   726
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   727
  "rtrancl''' (x, (x, x), r)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   728
| "r (x, y) ==> rtrancl''' (y, (z, z), r) ==> rtrancl''' (x, (z, z), r)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   729
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   730
code_pred rtrancl''' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   731
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   732
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   733
inductive succ :: "nat \<Rightarrow> nat \<Rightarrow> bool" where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   734
    "succ 0 1"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   735
  | "succ m n \<Longrightarrow> succ (Suc m) (Suc n)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   736
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   737
code_pred (modes: i => i => bool, i => o => bool, o => i => bool, o => o => bool) succ .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   738
code_pred [random_dseq] succ .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   739
thm succ.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   740
thm succ.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   741
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   742
values 10 "{(m, n). succ n m}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   743
values "{m. succ 0 m}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   744
values "{m. succ m 0}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   745
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   746
text \<open>values command needs mode annotation of the parameter succ
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   747
to disambiguate which mode is to be chosen.\<close> 
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   748
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   749
values [mode: i => o => bool] 20 "{n. tranclp succ 10 n}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   750
values [mode: o => i => bool] 10 "{n. tranclp succ n 10}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   751
values 20 "{(n, m). tranclp succ n m}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   752
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   753
inductive example_graph :: "int => int => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   754
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   755
  "example_graph 0 1"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   756
| "example_graph 1 2"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   757
| "example_graph 1 3"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   758
| "example_graph 4 7"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   759
| "example_graph 4 5"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   760
| "example_graph 5 6"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   761
| "example_graph 7 6"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   762
| "example_graph 7 8"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   763
 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   764
inductive not_reachable_in_example_graph :: "int => int => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   765
where "\<not> (tranclp example_graph x y) ==> not_reachable_in_example_graph x y"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   766
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   767
code_pred (expected_modes: i => i => bool) not_reachable_in_example_graph .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   768
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   769
thm not_reachable_in_example_graph.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   770
thm tranclp.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   771
value "not_reachable_in_example_graph 0 3"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   772
value "not_reachable_in_example_graph 4 8"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   773
value "not_reachable_in_example_graph 5 6"
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   774
text \<open>rtrancl compilation is strange!\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   775
(*
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   776
value "not_reachable_in_example_graph 0 4"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   777
value "not_reachable_in_example_graph 1 6"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   778
value "not_reachable_in_example_graph 8 4"*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   779
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   780
code_pred [dseq] not_reachable_in_example_graph .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   781
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   782
values [dseq 6] "{x. tranclp example_graph 0 3}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   783
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   784
values [dseq 0] "{x. not_reachable_in_example_graph 0 3}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   785
values [dseq 0] "{x. not_reachable_in_example_graph 0 4}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   786
values [dseq 20] "{x. not_reachable_in_example_graph 0 4}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   787
values [dseq 6] "{x. not_reachable_in_example_graph 0 3}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   788
values [dseq 3] "{x. not_reachable_in_example_graph 4 2}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   789
values [dseq 6] "{x. not_reachable_in_example_graph 4 2}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   790
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   791
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   792
inductive not_reachable_in_example_graph' :: "int => int => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   793
where "\<not> (rtranclp example_graph x y) ==> not_reachable_in_example_graph' x y"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   794
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   795
code_pred not_reachable_in_example_graph' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   796
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   797
value "not_reachable_in_example_graph' 0 3"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   798
(* value "not_reachable_in_example_graph' 0 5" would not terminate *)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   799
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   800
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   801
(*values [depth_limited 0] "{x. not_reachable_in_example_graph' 0 3}"*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   802
(*values [depth_limited 3] "{x. not_reachable_in_example_graph' 0 3}"*) (* fails with undefined *)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   803
(*values [depth_limited 5] "{x. not_reachable_in_example_graph' 0 3}"*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   804
(*values [depth_limited 1] "{x. not_reachable_in_example_graph' 0 4}"*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   805
(*values [depth_limit = 4] "{x. not_reachable_in_example_graph' 0 4}"*) (* fails with undefined *)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   806
(*values [depth_limit = 20] "{x. not_reachable_in_example_graph' 0 4}"*) (* fails with undefined *)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   807
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   808
code_pred [dseq] not_reachable_in_example_graph' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   809
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   810
(*thm not_reachable_in_example_graph'.dseq_equation*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   811
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   812
(*values [dseq 0] "{x. not_reachable_in_example_graph' 0 3}"*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   813
(*values [depth_limited 3] "{x. not_reachable_in_example_graph' 0 3}"*) (* fails with undefined *)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   814
(*values [depth_limited 5] "{x. not_reachable_in_example_graph' 0 3}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   815
values [depth_limited 1] "{x. not_reachable_in_example_graph' 0 4}"*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   816
(*values [depth_limit = 4] "{x. not_reachable_in_example_graph' 0 4}"*) (* fails with undefined *)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   817
(*values [depth_limit = 20] "{x. not_reachable_in_example_graph' 0 4}"*) (* fails with undefined *)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   818
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   819
subsection \<open>Free function variable\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   820
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   821
inductive FF :: "nat => nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   822
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   823
  "f x = y ==> FF x y"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   824
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   825
code_pred FF .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   826
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   827
subsection \<open>IMP\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   828
42463
f270e3e18be5 modernized specifications;
wenzelm
parents: 42208
diff changeset
   829
type_synonym var = nat
f270e3e18be5 modernized specifications;
wenzelm
parents: 42208
diff changeset
   830
type_synonym state = "int list"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   831
58310
91ea607a34d8 updated news
blanchet
parents: 58249
diff changeset
   832
datatype com =
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   833
  Skip |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   834
  Ass var "state => int" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   835
  Seq com com |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   836
  IF "state => bool" com com |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   837
  While "state => bool" com
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   838
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   839
inductive tupled_exec :: "(com \<times> state \<times> state) \<Rightarrow> bool" where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   840
"tupled_exec (Skip, s, s)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   841
"tupled_exec (Ass x e, s, s[x := e(s)])" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   842
"tupled_exec (c1, s1, s2) ==> tupled_exec (c2, s2, s3) ==> tupled_exec (Seq c1 c2, s1, s3)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   843
"b s ==> tupled_exec (c1, s, t) ==> tupled_exec (IF b c1 c2, s, t)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   844
"~b s ==> tupled_exec (c2, s, t) ==> tupled_exec (IF b c1 c2, s, t)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   845
"~b s ==> tupled_exec (While b c, s, s)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   846
"b s1 ==> tupled_exec (c, s1, s2) ==> tupled_exec (While b c, s2, s3) ==> tupled_exec (While b c, s1, s3)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   847
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   848
code_pred tupled_exec .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   849
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   850
values "{s. tupled_exec (While (%s. s!0 > 0) (Seq (Ass 0 (%s. s!0 - 1)) (Ass 1 (%s. s!1 + 1))), [3, 5], s)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   851
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   852
subsection \<open>CCS\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   853
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   854
text\<open>This example formalizes finite CCS processes without communication or
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   855
recursion. For simplicity, labels are natural numbers.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   856
58310
91ea607a34d8 updated news
blanchet
parents: 58249
diff changeset
   857
datatype proc = nil | pre nat proc | or proc proc | par proc proc
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   858
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   859
inductive tupled_step :: "(proc \<times> nat \<times> proc) \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   860
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   861
"tupled_step (pre n p, n, p)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   862
"tupled_step (p1, a, q) \<Longrightarrow> tupled_step (or p1 p2, a, q)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   863
"tupled_step (p2, a, q) \<Longrightarrow> tupled_step (or p1 p2, a, q)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   864
"tupled_step (p1, a, q) \<Longrightarrow> tupled_step (par p1 p2, a, par q p2)" |
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   865
"tupled_step (p2, a, q) \<Longrightarrow> tupled_step (par p1 p2, a, par p1 q)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   866
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   867
code_pred tupled_step .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   868
thm tupled_step.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   869
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   870
subsection \<open>divmod\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   871
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   872
inductive divmod_rel :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> bool" where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   873
    "k < l \<Longrightarrow> divmod_rel k l 0 k"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   874
  | "k \<ge> l \<Longrightarrow> divmod_rel (k - l) l q r \<Longrightarrow> divmod_rel k l (Suc q) r"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   875
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   876
code_pred divmod_rel .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   877
thm divmod_rel.equation
56927
4044a7d1720f hardcoded nbe and sml into value command
haftmann
parents: 56679
diff changeset
   878
value "Predicate.the (divmod_rel_i_i_o_o 1705 42)"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   879
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   880
subsection \<open>Transforming predicate logic into logic programs\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   881
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   882
subsection \<open>Transforming functions into logic programs\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   883
definition
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   884
  "case_f xs ys = (case (xs @ ys) of [] => [] | (x # xs) => xs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   885
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   886
code_pred [inductify, skip_proof] case_f .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   887
thm case_fP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   888
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   889
fun fold_map_idx where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   890
  "fold_map_idx f i y [] = (y, [])"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   891
| "fold_map_idx f i y (x # xs) =
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   892
 (let (y', x') = f i y x; (y'', xs') = fold_map_idx f (Suc i) y' xs
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   893
 in (y'', x' # xs'))"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   894
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   895
code_pred [inductify] fold_map_idx .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   896
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   897
subsection \<open>Minimum\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   898
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   899
definition Min
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   900
where "Min s r x \<equiv> s x \<and> (\<forall>y. r x y \<longrightarrow> x = y)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   901
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   902
code_pred [inductify] Min .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   903
thm Min.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   904
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   905
subsection \<open>Lexicographic order\<close>
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   906
text \<open>This example requires to handle the differences of sets and predicates in the predicate compiler,
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
   907
or to have a copy of all definitions on predicates due to the set-predicate distinction.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   908
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   909
(*
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   910
declare lexord_def[code_pred_def]
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   911
code_pred [inductify] lexord .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   912
code_pred [random_dseq inductify] lexord .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   913
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   914
thm lexord.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   915
thm lexord.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   916
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   917
inductive less_than_nat :: "nat * nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   918
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   919
  "less_than_nat (0, x)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   920
| "less_than_nat (x, y) ==> less_than_nat (Suc x, Suc y)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   921
 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   922
code_pred less_than_nat .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   923
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   924
code_pred [dseq] less_than_nat .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   925
code_pred [random_dseq] less_than_nat .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   926
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   927
inductive test_lexord :: "nat list * nat list => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   928
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   929
  "lexord less_than_nat (xs, ys) ==> test_lexord (xs, ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   930
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   931
code_pred test_lexord .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   932
code_pred [dseq] test_lexord .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   933
code_pred [random_dseq] test_lexord .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   934
thm test_lexord.dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   935
thm test_lexord.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   936
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   937
values "{x. test_lexord ([1, 2, 3], [1, 2, 5])}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   938
(*values [depth_limited 5] "{x. test_lexord ([1, 2, 3], [1, 2, 5])}"*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   939
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   940
lemmas [code_pred_def] = lexn_conv lex_conv lenlex_conv
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   941
(*
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   942
code_pred [inductify] lexn .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   943
thm lexn.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   944
*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   945
(*
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   946
code_pred [random_dseq inductify] lexn .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   947
thm lexn.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   948
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   949
values [random_dseq 4, 4, 6] 100 "{(n, xs, ys::int list). lexn (%(x, y). x <= y) n (xs, ys)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   950
*)
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
   951
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   952
inductive has_length
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   953
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   954
  "has_length [] 0"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   955
| "has_length xs i ==> has_length (x # xs) (Suc i)" 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   956
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   957
lemma has_length:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   958
  "has_length xs n = (length xs = n)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   959
proof (rule iffI)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   960
  assume "has_length xs n"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   961
  from this show "length xs = n"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   962
    by (rule has_length.induct) auto
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   963
next
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   964
  assume "length xs = n"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   965
  from this show "has_length xs n"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   966
    by (induct xs arbitrary: n) (auto intro: has_length.intros)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   967
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   968
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   969
lemma lexn_intros [code_pred_intro]:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   970
  "has_length xs i ==> has_length ys i ==> r (x, y) ==> lexn r (Suc i) (x # xs, y # ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   971
  "lexn r i (xs, ys) ==> lexn r (Suc i) (x # xs, x # ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   972
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   973
  assume "has_length xs i" "has_length ys i" "r (x, y)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   974
  from this has_length show "lexn r (Suc i) (x # xs, y # ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   975
    unfolding lexn_conv Collect_def mem_def
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42463
diff changeset
   976
    by fastforce
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   977
next
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   978
  assume "lexn r i (xs, ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   979
  thm lexn_conv
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   980
  from this show "lexn r (Suc i) (x#xs, x#ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   981
    unfolding Collect_def mem_def lexn_conv
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   982
    apply auto
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   983
    apply (rule_tac x="x # xys" in exI)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   984
    by auto
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   985
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   986
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   987
code_pred [random_dseq] lexn
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   988
proof -
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   989
  fix r n xs ys
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   990
  assume 1: "lexn r n (xs, ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   991
  assume 2: "\<And>r' i x xs' y ys'. r = r' ==> n = Suc i ==> (xs, ys) = (x # xs', y # ys') ==> has_length xs' i ==> has_length ys' i ==> r' (x, y) ==> thesis"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   992
  assume 3: "\<And>r' i x xs' ys'. r = r' ==> n = Suc i ==> (xs, ys) = (x # xs', x # ys') ==> lexn r' i (xs', ys') ==> thesis"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   993
  from 1 2 3 show thesis
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   994
    unfolding lexn_conv Collect_def mem_def
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   995
    apply (auto simp add: has_length)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   996
    apply (case_tac xys)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
   997
    apply auto
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42463
diff changeset
   998
    apply fastforce
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42463
diff changeset
   999
    apply fastforce done
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1000
qed
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1001
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1002
values [random_dseq 1, 2, 5] 10 "{(n, xs, ys::int list). lexn (%(x, y). x <= y) n (xs, ys)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1003
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1004
code_pred [inductify, skip_proof] lex .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1005
thm lex.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1006
thm lex_def
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1007
declare lenlex_conv[code_pred_def]
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1008
code_pred [inductify, skip_proof] lenlex .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1009
thm lenlex.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1010
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1011
code_pred [random_dseq inductify] lenlex .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1012
thm lenlex.random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1013
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1014
values [random_dseq 4, 2, 4] 100 "{(xs, ys::int list). lenlex (%(x, y). x <= y) (xs, ys)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1015
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1016
thm lists.intros
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1017
code_pred [inductify] lists .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1018
thm lists.equation
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1019
*)
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1020
subsection \<open>AVL Tree\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1021
58310
91ea607a34d8 updated news
blanchet
parents: 58249
diff changeset
  1022
datatype 'a tree = ET | MKT 'a "'a tree" "'a tree" nat
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1023
fun height :: "'a tree => nat" where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1024
"height ET = 0"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1025
| "height (MKT x l r h) = max (height l) (height r) + 1"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1026
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1027
primrec avl :: "'a tree => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1028
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1029
  "avl ET = True"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1030
| "avl (MKT x l r h) = ((height l = height r \<or> height l = 1 + height r \<or> height r = 1+height l) \<and> 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1031
  h = max (height l) (height r) + 1 \<and> avl l \<and> avl r)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1032
(*
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1033
code_pred [inductify] avl .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1034
thm avl.equation*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1035
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1036
code_pred [new_random_dseq inductify] avl .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1037
thm avl.new_random_dseq_equation
40137
9eabcb1bfe50 changing test parameters in examples to get to a result within the global timelimit
bulwahn
parents: 40100
diff changeset
  1038
(* TODO: has highly non-deterministic execution time!
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1039
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1040
values [new_random_dseq 2, 1, 7] 5 "{t:: int tree. avl t}"
40137
9eabcb1bfe50 changing test parameters in examples to get to a result within the global timelimit
bulwahn
parents: 40100
diff changeset
  1041
*)
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1042
fun set_of
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1043
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1044
"set_of ET = {}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1045
| "set_of (MKT n l r h) = insert n (set_of l \<union> set_of r)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1046
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1047
fun is_ord :: "nat tree => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1048
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1049
"is_ord ET = True"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1050
| "is_ord (MKT n l r h) =
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1051
 ((\<forall>n' \<in> set_of l. n' < n) \<and> (\<forall>n' \<in> set_of r. n < n') \<and> is_ord l \<and> is_ord r)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1052
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1053
(* 
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1054
code_pred (expected_modes: i => o => bool, i => i => bool) [inductify] set_of .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1055
thm set_of.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1056
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1057
code_pred (expected_modes: i => bool) [inductify] is_ord .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1058
thm is_ord_aux.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1059
thm is_ord.equation
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1060
*)
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1061
subsection \<open>Definitions about Relations\<close>
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1062
(*
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1063
code_pred (modes:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1064
  (i * i => bool) => i * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1065
  (i * o => bool) => o * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1066
  (i * o => bool) => i * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1067
  (o * i => bool) => i * o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1068
  (o * i => bool) => i * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1069
  (o * o => bool) => o * o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1070
  (o * o => bool) => i * o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1071
  (o * o => bool) => o * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1072
  (o * o => bool) => i * i => bool) [inductify] converse .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1073
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1074
thm converse.equation
47433
07f4bf913230 renamed "rel_comp" to "relcomp" (to be consistent with, e.g., "relpow")
griff
parents: 47108
diff changeset
  1075
code_pred [inductify] relcomp .
07f4bf913230 renamed "rel_comp" to "relcomp" (to be consistent with, e.g., "relpow")
griff
parents: 47108
diff changeset
  1076
thm relcomp.equation
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1077
code_pred [inductify] Image .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1078
thm Image.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1079
declare singleton_iff[code_pred_inline]
44928
7ef6505bde7f renamed Complete_Lattices lemmas, removed legacy names
hoelzl
parents: 44890
diff changeset
  1080
declare Id_on_def[unfolded Bex_def UNION_eq singleton_iff, code_pred_def]
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1081
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1082
code_pred (expected_modes:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1083
  (o => bool) => o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1084
  (o => bool) => i * o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1085
  (o => bool) => o * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1086
  (o => bool) => i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1087
  (i => bool) => i * o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1088
  (i => bool) => o * i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1089
  (i => bool) => i => bool) [inductify] Id_on .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1090
thm Id_on.equation
46752
e9e7209eb375 more fundamental pred-to-set conversions, particularly by means of inductive_set; associated consolidation of some theorem names (c.f. NEWS)
haftmann
parents: 45970
diff changeset
  1091
thm Domain_unfold
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1092
code_pred (modes:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1093
  (o * o => bool) => o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1094
  (o * o => bool) => i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1095
  (i * o => bool) => i => bool) [inductify] Domain .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1096
thm Domain.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1097
46752
e9e7209eb375 more fundamental pred-to-set conversions, particularly by means of inductive_set; associated consolidation of some theorem names (c.f. NEWS)
haftmann
parents: 45970
diff changeset
  1098
thm Domain_converse [symmetric]
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1099
code_pred (modes:
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1100
  (o * o => bool) => o => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1101
  (o * o => bool) => i => bool,
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1102
  (o * i => bool) => i => bool) [inductify] Range .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1103
thm Range.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1104
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1105
code_pred [inductify] Field .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1106
thm Field.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1107
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1108
thm refl_on_def
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1109
code_pred [inductify] refl_on .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1110
thm refl_on.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1111
code_pred [inductify] total_on .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1112
thm total_on.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1113
code_pred [inductify] antisym .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1114
thm antisym.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1115
code_pred [inductify] trans .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1116
thm trans.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1117
code_pred [inductify] single_valued .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1118
thm single_valued.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1119
thm inv_image_def
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1120
code_pred [inductify] inv_image .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1121
thm inv_image.equation
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1122
*)
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1123
subsection \<open>Inverting list functions\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1124
56679
5545bfdfefcc avoid name shadowing
blanchet
parents: 55932
diff changeset
  1125
code_pred [inductify, skip_proof] size_list' .
5545bfdfefcc avoid name shadowing
blanchet
parents: 55932
diff changeset
  1126
code_pred [new_random_dseq inductify] size_list' .
5545bfdfefcc avoid name shadowing
blanchet
parents: 55932
diff changeset
  1127
thm size_list'P.equation
5545bfdfefcc avoid name shadowing
blanchet
parents: 55932
diff changeset
  1128
thm size_list'P.new_random_dseq_equation
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1129
56679
5545bfdfefcc avoid name shadowing
blanchet
parents: 55932
diff changeset
  1130
values [new_random_dseq 2,3,10] 3 "{xs. size_list'P (xs::nat list) (5::nat)}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1131
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1132
code_pred (expected_modes: i => o => bool, o => i => bool, i => i => bool) [inductify, skip_proof] List.concat .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1133
thm concatP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1134
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1135
values "{ys. concatP [[1, 2], [3, (4::int)]] ys}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1136
values "{ys. concatP [[1, 2], [3]] [1, 2, (3::nat)]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1137
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1138
code_pred [dseq inductify] List.concat .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1139
thm concatP.dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1140
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1141
values [dseq 3] 3
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1142
  "{xs. concatP xs ([0] :: nat list)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1143
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1144
values [dseq 5] 3
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1145
  "{xs. concatP xs ([1] :: int list)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1146
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1147
values [dseq 5] 3
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1148
  "{xs. concatP xs ([1] :: nat list)}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1149
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1150
values [dseq 5] 3
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1151
  "{xs. concatP xs [(1::int), 2]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1152
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1153
code_pred (expected_modes: i => o => bool, i => i => bool) [inductify] hd .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1154
thm hdP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1155
values "{x. hdP [1, 2, (3::int)] x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1156
values "{(xs, x). hdP [1, 2, (3::int)] 1}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1157
 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1158
code_pred (expected_modes: i => o => bool, i => i => bool) [inductify] tl .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1159
thm tlP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1160
values "{x. tlP [1, 2, (3::nat)] x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1161
values "{x. tlP [1, 2, (3::int)] [3]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1162
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1163
code_pred [inductify, skip_proof] last .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1164
thm lastP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1165
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1166
code_pred [inductify, skip_proof] butlast .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1167
thm butlastP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1168
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1169
code_pred [inductify, skip_proof] take .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1170
thm takeP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1171
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1172
code_pred [inductify, skip_proof] drop .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1173
thm dropP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1174
code_pred [inductify, skip_proof] zip .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1175
thm zipP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1176
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1177
code_pred [inductify, skip_proof] upt .
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1178
(*
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1179
code_pred [inductify, skip_proof] remdups .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1180
thm remdupsP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1181
code_pred [dseq inductify] remdups .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1182
values [dseq 4] 5 "{xs. remdupsP xs [1, (2::int)]}"
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1183
*)
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1184
code_pred [inductify, skip_proof] remove1 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1185
thm remove1P.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1186
values "{xs. remove1P 1 xs [2, (3::int)]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1187
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1188
code_pred [inductify, skip_proof] removeAll .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1189
thm removeAllP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1190
code_pred [dseq inductify] removeAll .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1191
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1192
values [dseq 4] 10 "{xs. removeAllP 1 xs [(2::nat)]}"
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1193
(*
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1194
code_pred [inductify] distinct .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1195
thm distinct.equation
45970
b6d0cff57d96 adjusted to set/pred distinction by means of type constructor `set`
haftmann
parents: 44928
diff changeset
  1196
*)
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1197
code_pred [inductify, skip_proof] replicate .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1198
thm replicateP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1199
values 5 "{(n, xs). replicateP n (0::int) xs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1200
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1201
code_pred [inductify, skip_proof] splice .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1202
thm splice.simps
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1203
thm spliceP.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1204
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1205
values "{xs. spliceP xs [1, 2, 3] [1, 1, 1, 2, 1, (3::nat)]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1206
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1207
code_pred [inductify, skip_proof] List.rev .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1208
code_pred [inductify] map .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1209
code_pred [inductify] foldr .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1210
code_pred [inductify] foldl .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1211
code_pred [inductify] filter .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1212
code_pred [random_dseq inductify] filter .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1213
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1214
section \<open>Function predicate replacement\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1215
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1216
text \<open>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1217
If the mode analysis uses the functional mode, we
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1218
replace predicates that resulted from functions again by their functions.
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1219
\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1220
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1221
inductive test_append
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1222
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1223
  "List.append xs ys = zs ==> test_append xs ys zs"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1224
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1225
code_pred [inductify, skip_proof] test_append .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1226
thm test_append.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1227
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1228
text \<open>If append is not turned into a predicate, then the mode
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1229
  o => o => i => bool could not be inferred.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1230
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1231
values 4 "{(xs::int list, ys). test_append xs ys [1, 2, 3, 4]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1232
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1233
text \<open>If appendP is not reverted back to a function, then mode i => i => o => bool
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1234
  fails after deleting the predicate equation.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1235
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1236
declare appendP.equation[code del]
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1237
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1238
values "{xs::int list. test_append [1,2] [3,4] xs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1239
values "{xs::int list. test_append (replicate 1000 1) (replicate 1000 2) xs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1240
values "{xs::int list. test_append (replicate 2000 1) (replicate 2000 2) xs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1241
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1242
text \<open>Redeclaring append.equation as code equation\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1243
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1244
declare appendP.equation[code]
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1245
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1246
subsection \<open>Function with tuples\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1247
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1248
fun append'
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1249
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1250
  "append' ([], ys) = ys"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1251
| "append' (x # xs, ys) = x # append' (xs, ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1252
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1253
inductive test_append'
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1254
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1255
  "append' (xs, ys) = zs ==> test_append' xs ys zs"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1256
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1257
code_pred [inductify, skip_proof] test_append' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1258
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1259
thm test_append'.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1260
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1261
values "{(xs::int list, ys). test_append' xs ys [1, 2, 3, 4]}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1262
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1263
declare append'P.equation[code del]
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1264
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1265
values "{zs :: int list. test_append' [1,2,3] [4,5] zs}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1266
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1267
section \<open>Arithmetic examples\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1268
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1269
subsection \<open>Examples on nat\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1270
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1271
inductive plus_nat_test :: "nat => nat => nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1272
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1273
  "x + y = z ==> plus_nat_test x y z"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1274
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1275
code_pred [inductify, skip_proof] plus_nat_test .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1276
code_pred [new_random_dseq inductify] plus_nat_test .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1277
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1278
thm plus_nat_test.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1279
thm plus_nat_test.new_random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1280
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1281
values [expected "{9::nat}"] "{z. plus_nat_test 4 5 z}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1282
values [expected "{9::nat}"] "{z. plus_nat_test 7 2 z}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1283
values [expected "{4::nat}"] "{y. plus_nat_test 5 y 9}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1284
values [expected "{}"] "{y. plus_nat_test 9 y 8}"
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1285
values [expected "{6::nat}"] "{y. plus_nat_test 1 y 7}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1286
values [expected "{2::nat}"] "{x. plus_nat_test x 7 9}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1287
values [expected "{}"] "{x. plus_nat_test x 9 7}"
51144
0ede9e2266a8 less customary term_of conversions;
haftmann
parents: 51143
diff changeset
  1288
values [expected "{(0::nat, 0::nat)}"] "{(x, y). plus_nat_test x y 0}"
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1289
values [expected "{(0, 1), (1::nat, 0::nat)}"] "{(x, y). plus_nat_test x y 1}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1290
values [expected "{(0::nat, 5::nat), (1, 4), (2, 3), (3, 2), (4, 1), (5, 0)}"]
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1291
  "{(x, y). plus_nat_test x y 5}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1292
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1293
inductive minus_nat_test :: "nat => nat => nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1294
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1295
  "x - y = z ==> minus_nat_test x y z"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1296
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1297
code_pred [inductify, skip_proof] minus_nat_test .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1298
code_pred [new_random_dseq inductify] minus_nat_test .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1299
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1300
thm minus_nat_test.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1301
thm minus_nat_test.new_random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1302
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1303
values [expected "{0::nat}"] "{z. minus_nat_test 4 5 z}"
66283
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1304
values [expected "{5::nat}"] "{z. minus_nat_test 7 2 z}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1305
values [expected "{16::nat}"] "{x. minus_nat_test x 7 9}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1306
values [expected "{16::nat}"] "{x. minus_nat_test x 9 7}"
adf3155c57e2 Printing natural numbers as numerals in evaluation
eberlm <eberlm@in.tum.de>
parents: 64542
diff changeset
  1307
values [expected "{0::nat, 1, 2, 3}"] "{x. minus_nat_test x 3 0}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1308
values [expected "{0::nat}"] "{x. minus_nat_test x 0 0}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1309
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1310
subsection \<open>Examples on int\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1311
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1312
inductive plus_int_test :: "int => int => int => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1313
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1314
  "a + b = c ==> plus_int_test a b c"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1315
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1316
code_pred [inductify, skip_proof] plus_int_test .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1317
code_pred [new_random_dseq inductify] plus_int_test .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1318
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1319
thm plus_int_test.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1320
thm plus_int_test.new_random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1321
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1322
values [expected "{1::int}"] "{a. plus_int_test a 6 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1323
values [expected "{1::int}"] "{b. plus_int_test 6 b 7}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1324
values [expected "{11::int}"] "{c. plus_int_test 5 6 c}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1325
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1326
inductive minus_int_test :: "int => int => int => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1327
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1328
  "a - b = c ==> minus_int_test a b c"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1329
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1330
code_pred [inductify, skip_proof] minus_int_test .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1331
code_pred [new_random_dseq inductify] minus_int_test .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1332
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1333
thm minus_int_test.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1334
thm minus_int_test.new_random_dseq_equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1335
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1336
values [expected "{4::int}"] "{c. minus_int_test 9 5 c}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1337
values [expected "{9::int}"] "{a. minus_int_test a 4 5}"
40885
da4bdafeef7c adapted expected value to more idiomatic numeral representation
haftmann
parents: 40137
diff changeset
  1338
values [expected "{-1::int}"] "{b. minus_int_test 4 b 5}"
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1339
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1340
subsection \<open>minus on bool\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1341
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1342
inductive All :: "nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1343
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1344
  "All x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1345
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1346
inductive None :: "nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1347
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1348
definition "test_minus_bool x = (None x - All x)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1349
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1350
code_pred [inductify] test_minus_bool .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1351
thm test_minus_bool.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1352
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1353
values "{x. test_minus_bool x}"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1354
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1355
subsection \<open>Functions\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1356
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1357
fun partial_hd :: "'a list => 'a option"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1358
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1359
  "partial_hd [] = Option.None"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1360
| "partial_hd (x # xs) = Some x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1361
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1362
inductive hd_predicate
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1363
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1364
  "partial_hd xs = Some x ==> hd_predicate xs x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1365
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1366
code_pred (expected_modes: i => i => bool, i => o => bool) hd_predicate .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1367
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1368
thm hd_predicate.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1369
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1370
subsection \<open>Locales\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1371
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1372
inductive hd_predicate2 :: "('a list => 'a option) => 'a list => 'a => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1373
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1374
  "partial_hd' xs = Some x ==> hd_predicate2 partial_hd' xs x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1375
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1376
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1377
thm hd_predicate2.intros
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1378
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1379
code_pred (expected_modes: i => i => i => bool, i => i => o => bool) hd_predicate2 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1380
thm hd_predicate2.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1381
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1382
locale A = fixes partial_hd :: "'a list => 'a option" begin
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1383
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1384
inductive hd_predicate_in_locale :: "'a list => 'a => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1385
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1386
  "partial_hd xs = Some x ==> hd_predicate_in_locale xs x"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1387
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1388
end
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1389
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1390
text \<open>The global introduction rules must be redeclared as introduction rules and then 
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1391
  one could invoke code_pred.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1392
39657
5e57675b7e40 moving the preprocessing of introduction rules after the code_pred command; added tuple expansion preprocessing of elimination rule
bulwahn
parents: 39655
diff changeset
  1393
declare A.hd_predicate_in_locale.intros [code_pred_intro]
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1394
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1395
code_pred (expected_modes: i => i => i => bool, i => i => o => bool) A.hd_predicate_in_locale
39657
5e57675b7e40 moving the preprocessing of introduction rules after the code_pred command; added tuple expansion preprocessing of elimination rule
bulwahn
parents: 39655
diff changeset
  1396
by (auto elim: A.hd_predicate_in_locale.cases)
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1397
    
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1398
interpretation A partial_hd .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1399
thm hd_predicate_in_locale.intros
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1400
text \<open>A locally compliant solution with a trivial interpretation fails, because
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1401
the predicate compiler has very strict assumptions about the terms and their structure.\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1402
 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1403
(*code_pred hd_predicate_in_locale .*)
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1404
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1405
section \<open>Integer example\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1406
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1407
definition three :: int
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1408
where "three = 3"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1409
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1410
inductive is_three
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1411
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1412
  "is_three three"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1413
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1414
code_pred is_three .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1415
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1416
thm is_three.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1417
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1418
section \<open>String.literal example\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1419
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1420
definition Error_1
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1421
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1422
  "Error_1 = STR ''Error 1''"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1423
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1424
definition Error_2
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1425
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1426
  "Error_2 = STR ''Error 2''"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1427
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1428
inductive "is_error" :: "String.literal \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1429
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1430
  "is_error Error_1"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1431
| "is_error Error_2"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1432
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1433
code_pred is_error .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1434
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1435
thm is_error.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1436
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1437
inductive is_error' :: "String.literal \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1438
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1439
  "is_error' (STR ''Error1'')"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1440
| "is_error' (STR ''Error2'')"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1441
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1442
code_pred is_error' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1443
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1444
thm is_error'.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1445
58310
91ea607a34d8 updated news
blanchet
parents: 58249
diff changeset
  1446
datatype ErrorObject = Error String.literal int
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1447
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1448
inductive is_error'' :: "ErrorObject \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1449
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1450
  "is_error'' (Error Error_1 3)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1451
| "is_error'' (Error Error_2 4)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1452
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1453
code_pred is_error'' .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1454
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1455
thm is_error''.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1456
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1457
section \<open>Another function example\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1458
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1459
consts f :: "'a \<Rightarrow> 'a"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1460
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1461
inductive fun_upd :: "(('a * 'b) * ('a \<Rightarrow> 'b)) \<Rightarrow> ('a \<Rightarrow> 'b) \<Rightarrow> bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1462
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1463
  "fun_upd ((x, a), s) (s(x := f a))"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1464
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1465
code_pred fun_upd .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1466
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1467
thm fun_upd.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1468
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1469
section \<open>Examples for detecting switches\<close>
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1470
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1471
inductive detect_switches1 where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1472
  "detect_switches1 [] []"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1473
| "detect_switches1 (x # xs) (y # ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1474
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1475
code_pred [detect_switches, skip_proof] detect_switches1 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1476
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1477
thm detect_switches1.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1478
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1479
inductive detect_switches2 :: "('a => bool) => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1480
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1481
  "detect_switches2 P"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1482
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1483
code_pred [detect_switches, skip_proof] detect_switches2 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1484
thm detect_switches2.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1485
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1486
inductive detect_switches3 :: "('a => bool) => 'a list => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1487
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1488
  "detect_switches3 P []"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1489
| "detect_switches3 P (x # xs)" 
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1490
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1491
code_pred [detect_switches, skip_proof] detect_switches3 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1492
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1493
thm detect_switches3.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1494
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1495
inductive detect_switches4 :: "('a => bool) => 'a list => 'a list => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1496
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1497
  "detect_switches4 P [] []"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1498
| "detect_switches4 P (x # xs) (y # ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1499
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1500
code_pred [detect_switches, skip_proof] detect_switches4 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1501
thm detect_switches4.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1502
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1503
inductive detect_switches5 :: "('a => 'a => bool) => 'a list => 'a list => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1504
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1505
  "detect_switches5 P [] []"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1506
| "detect_switches5 P xs ys ==> P x y ==> detect_switches5 P (x # xs) (y # ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1507
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1508
code_pred [detect_switches, skip_proof] detect_switches5 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1509
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1510
thm detect_switches5.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1511
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1512
inductive detect_switches6 :: "(('a => 'b => bool) * 'a list * 'b list) => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1513
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1514
  "detect_switches6 (P, [], [])"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1515
| "detect_switches6 (P, xs, ys) ==> P x y ==> detect_switches6 (P, x # xs, y # ys)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1516
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1517
code_pred [detect_switches, skip_proof] detect_switches6 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1518
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1519
inductive detect_switches7 :: "('a => bool) => ('b => bool) => ('a * 'b list) => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1520
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1521
  "detect_switches7 P Q (a, [])"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1522
| "P a ==> Q x ==> detect_switches7 P Q (a, x#xs)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1523
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1524
code_pred [skip_proof] detect_switches7 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1525
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1526
thm detect_switches7.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1527
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1528
inductive detect_switches8 :: "nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1529
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1530
  "detect_switches8 0"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1531
| "x mod 2 = 0 ==> detect_switches8 (Suc x)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1532
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1533
code_pred [detect_switches, skip_proof] detect_switches8 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1534
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1535
thm detect_switches8.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1536
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1537
inductive detect_switches9 :: "nat => nat => bool"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1538
where
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1539
  "detect_switches9 0 0"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1540
| "detect_switches9 0 (Suc x)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1541
| "detect_switches9 (Suc x) 0"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1542
| "x = y ==> detect_switches9 (Suc x) (Suc y)"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1543
| "c1 = c2 ==> detect_switches9 c1 c2"
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1544
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1545
code_pred [detect_switches, skip_proof] detect_switches9 .
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1546
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1547
thm detect_switches9.equation
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1548
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1549
text \<open>The higher-order predicate r is in an output term\<close>
39762
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1550
58310
91ea607a34d8 updated news
blanchet
parents: 58249
diff changeset
  1551
datatype result = Result bool
39762
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1552
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1553
inductive fixed_relation :: "'a => bool"
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1554
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1555
inductive test_relation_in_output_terms :: "('a => bool) => 'a => result => bool"
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1556
where
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1557
  "test_relation_in_output_terms r x (Result (r x))"
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1558
| "test_relation_in_output_terms r x (Result (fixed_relation x))"
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1559
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1560
code_pred test_relation_in_output_terms .
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1561
02fb709ab3cb handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn
parents: 39657
diff changeset
  1562
thm test_relation_in_output_terms.equation
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1563
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1564
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1565
text \<open>
39765
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1566
  We want that the argument r is not treated as a higher-order relation, but simply as input.
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1567
\<close>
39765
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1568
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1569
inductive test_uninterpreted_relation :: "('a => bool) => 'a list => bool"
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1570
where
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1571
  "list_all r xs ==> test_uninterpreted_relation r xs"
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1572
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1573
code_pred (modes: i => i => bool) test_uninterpreted_relation .
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1574
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1575
thm test_uninterpreted_relation.equation
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1576
39786
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1577
inductive list_ex'
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1578
where
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1579
  "P x ==> list_ex' P (x#xs)"
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1580
| "list_ex' P xs ==> list_ex' P (x#xs)"
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1581
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1582
code_pred list_ex' .
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1583
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1584
inductive test_uninterpreted_relation2 :: "('a => bool) => 'a list => bool"
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1585
where
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1586
  "list_ex r xs ==> test_uninterpreted_relation2 r xs"
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1587
| "list_ex' r xs ==> test_uninterpreted_relation2 r xs"
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1588
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1589
text \<open>Proof procedure cannot handle this situation yet.\<close>
39786
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1590
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1591
code_pred (modes: i => i => bool) [skip_proof] test_uninterpreted_relation2 .
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1592
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1593
thm test_uninterpreted_relation2.equation
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1594
30c077288dfe added test case for predicate arguments in higher-order argument position
bulwahn
parents: 39784
diff changeset
  1595
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1596
text \<open>Trivial predicate\<close>
39784
cfd06840f477 added a test case to Predicate_Compile_Tests
bulwahn
parents: 39765
diff changeset
  1597
cfd06840f477 added a test case to Predicate_Compile_Tests
bulwahn
parents: 39765
diff changeset
  1598
inductive implies_itself :: "'a => bool"
cfd06840f477 added a test case to Predicate_Compile_Tests
bulwahn
parents: 39765
diff changeset
  1599
where
cfd06840f477 added a test case to Predicate_Compile_Tests
bulwahn
parents: 39765
diff changeset
  1600
  "implies_itself x ==> implies_itself x"
cfd06840f477 added a test case to Predicate_Compile_Tests
bulwahn
parents: 39765
diff changeset
  1601
cfd06840f477 added a test case to Predicate_Compile_Tests
bulwahn
parents: 39765
diff changeset
  1602
code_pred implies_itself .
39765
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1603
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 62121
diff changeset
  1604
text \<open>Case expressions\<close>
39803
a8178a7b7b51 adding example for case expressions
bulwahn
parents: 39786
diff changeset
  1605
a8178a7b7b51 adding example for case expressions
bulwahn
parents: 39786
diff changeset
  1606
definition
55932
68c5104d2204 renamed 'map_pair' to 'map_prod'
blanchet
parents: 51144
diff changeset
  1607
  "map_prods xs ys = (map (%((a, b), c). (a, b, c)) xs = ys)"
39803
a8178a7b7b51 adding example for case expressions
bulwahn
parents: 39786
diff changeset
  1608
55932
68c5104d2204 renamed 'map_pair' to 'map_prod'
blanchet
parents: 51144
diff changeset
  1609
code_pred [inductify] map_prods .
39765
19cb8d558166 adding test case for interpretation of arguments that are predicates simply as input
bulwahn
parents: 39762
diff changeset
  1610
39655
8ad7fe9d6f0b splitting Predicate_Compile_Examples into Examples and Predicate_Compile_Tests
bulwahn
parents:
diff changeset
  1611
end