author | haftmann |
Fri, 29 Dec 2006 12:11:00 +0100 | |
changeset 21924 | fe474e69e603 |
parent 20663 | 2024d9f7df9c |
child 23323 | 2274edb9a8b2 |
permissions | -rw-r--r-- |
13880 | 1 |
(* Title: HOL/ex/PresburgerEx.thy |
2 |
ID: $Id$ |
|
3 |
Author: Amine Chaieb, TU Muenchen |
|
17388 | 4 |
*) |
13880 | 5 |
|
17388 | 6 |
header {* Some examples for Presburger Arithmetic *} |
13880 | 7 |
|
16417 | 8 |
theory PresburgerEx imports Main begin |
13880 | 9 |
|
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
10 |
theorem "(\<forall>(y::int). 3 dvd y) ==> \<forall>(x::int). b < x --> a \<le> x" |
13880 | 11 |
by presburger |
12 |
||
13 |
theorem "!! (y::int) (z::int) (n::int). 3 dvd z ==> 2 dvd (y::int) ==> |
|
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
14 |
(\<exists>(x::int). 2*x = y) & (\<exists>(k::int). 3*k = z)" |
13880 | 15 |
by presburger |
16 |
||
17 |
theorem "!! (y::int) (z::int) n. Suc(n::nat) < 6 ==> 3 dvd z ==> |
|
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
18 |
2 dvd (y::int) ==> (\<exists>(x::int). 2*x = y) & (\<exists>(k::int). 3*k = z)" |
13880 | 19 |
by presburger |
20 |
||
15075 | 21 |
theorem "\<forall>(x::nat). \<exists>(y::nat). (0::nat) \<le> 5 --> y = 5 + x " |
13880 | 22 |
by presburger |
23 |
||
20663 | 24 |
text{*Slow: about 7 seconds on a 1.6GHz machine.*} |
15075 | 25 |
theorem "\<forall>(x::nat). \<exists>(y::nat). y = 5 + x | x div 6 + 1= 2" |
26 |
by presburger |
|
27 |
||
28 |
theorem "\<exists>(x::int). 0 < x" |
|
13880 | 29 |
by presburger |
30 |
||
15075 | 31 |
theorem "\<forall>(x::int) y. x < y --> 2 * x + 1 < 2 * y" |
32 |
by presburger |
|
13880 | 33 |
|
15075 | 34 |
theorem "\<forall>(x::int) y. 2 * x + 1 \<noteq> 2 * y" |
35 |
by presburger |
|
13880 | 36 |
|
15075 | 37 |
theorem "\<exists>(x::int) y. 0 < x & 0 \<le> y & 3 * x - 5 * y = 1" |
38 |
by presburger |
|
13880 | 39 |
|
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
40 |
theorem "~ (\<exists>(x::int) (y::int) (z::int). 4*x + (-6::int)*y = 1)" |
13880 | 41 |
by presburger |
42 |
||
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
43 |
theorem "\<forall>(x::int). b < x --> a \<le> x" |
14758
af3b71a46a1c
A new implementation for presburger arithmetic following the one suggested in technical report Chaieb Amine and Tobias Nipkow. It is generic an smaller.
chaieb
parents:
14353
diff
changeset
|
44 |
apply (presburger (no_quantify)) |
13880 | 45 |
oops |
46 |
||
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
47 |
theorem "~ (\<exists>(x::int). False)" |
13880 | 48 |
by presburger |
49 |
||
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
50 |
theorem "\<forall>(x::int). (a::int) < 3 * x --> b < 3 * x" |
14758
af3b71a46a1c
A new implementation for presburger arithmetic following the one suggested in technical report Chaieb Amine and Tobias Nipkow. It is generic an smaller.
chaieb
parents:
14353
diff
changeset
|
51 |
apply (presburger (no_quantify)) |
13880 | 52 |
oops |
53 |
||
15075 | 54 |
theorem "\<forall>(x::int). (2 dvd x) --> (\<exists>(y::int). x = 2*y)" |
55 |
by presburger |
|
13880 | 56 |
|
15075 | 57 |
theorem "\<forall>(x::int). (2 dvd x) --> (\<exists>(y::int). x = 2*y)" |
58 |
by presburger |
|
13880 | 59 |
|
15075 | 60 |
theorem "\<forall>(x::int). (2 dvd x) = (\<exists>(y::int). x = 2*y)" |
61 |
by presburger |
|
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
62 |
|
15075 | 63 |
theorem "\<forall>(x::int). ((2 dvd x) = (\<forall>(y::int). x \<noteq> 2*y + 1))" |
64 |
by presburger |
|
13880 | 65 |
|
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
66 |
theorem "~ (\<forall>(x::int). |
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
67 |
((2 dvd x) = (\<forall>(y::int). x \<noteq> 2*y+1) | |
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
68 |
(\<exists>(q::int) (u::int) i. 3*i + 2*q - u < 17) |
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
69 |
--> 0 < x | ((~ 3 dvd x) &(x + 8 = 0))))" |
13880 | 70 |
by presburger |
71 |
||
15075 | 72 |
theorem "~ (\<forall>(i::int). 4 \<le> i --> (\<exists>x y. 0 \<le> x & 0 \<le> y & 3 * x + 5 * y = i))" |
13880 | 73 |
by presburger |
74 |
||
15075 | 75 |
theorem "\<forall>(i::int). 8 \<le> i --> (\<exists>x y. 0 \<le> x & 0 \<le> y & 3 * x + 5 * y = i)" |
14353
79f9fbef9106
Added lemmas to Ring_and_Field with slightly modified simplification rules
paulson
parents:
13880
diff
changeset
|
76 |
by presburger |
13880 | 77 |
|
15075 | 78 |
theorem "\<exists>(j::int). \<forall>i. j \<le> i --> (\<exists>x y. 0 \<le> x & 0 \<le> y & 3 * x + 5 * y = i)" |
79 |
by presburger |
|
80 |
||
81 |
theorem "~ (\<forall>j (i::int). j \<le> i --> (\<exists>x y. 0 \<le> x & 0 \<le> y & 3 * x + 5 * y = i))" |
|
13880 | 82 |
by presburger |
83 |
||
20663 | 84 |
text{*Slow: about 5 seconds on a 1.6GHz machine.*} |
15075 | 85 |
theorem "(\<exists>m::nat. n = 2 * m) --> (n + 1) div 2 = n div 2" |
86 |
by presburger |
|
13880 | 87 |
|
19824 | 88 |
text{* This following theorem proves that all solutions to the |
89 |
recurrence relation $x_{i+2} = |x_{i+1}| - x_i$ are periodic with |
|
90 |
period 9. The example was brought to our attention by John |
|
91 |
Harrison. It does does not require Presburger arithmetic but merely |
|
92 |
quantifier-free linear arithmetic and holds for the rationals as well. |
|
93 |
||
20663 | 94 |
Warning: it takes (in 2006) over 4.2 minutes! *} |
19824 | 95 |
|
96 |
lemma "\<lbrakk> x3 = abs x2 - x1; x4 = abs x3 - x2; x5 = abs x4 - x3; |
|
97 |
x6 = abs x5 - x4; x7 = abs x6 - x5; x8 = abs x7 - x6; |
|
98 |
x9 = abs x8 - x7; x10 = abs x9 - x8; x11 = abs x10 - x9 \<rbrakk> |
|
99 |
\<Longrightarrow> x1 = x10 & x2 = (x11::int)" |
|
100 |
by arith |
|
101 |
||
15075 | 102 |
end |