author | huffman |
Sun, 09 May 2010 17:47:43 -0700 | |
changeset 36777 | be5461582d0f |
parent 35699 | 9ed327529a44 |
child 37495 | 650fae5eea93 |
permissions | -rw-r--r-- |
33197 | 1 |
(* Title: HOL/Nitpick_Examples/Mini_Nits.thy |
2 |
Author: Jasmin Blanchette, TU Muenchen |
|
35076
cc19e2aef17e
added hotel key card example for Nitpick, and renumber atoms in Nitpick's output for increased readability
blanchet
parents:
33197
diff
changeset
|
3 |
Copyright 2009, 2010 |
33197 | 4 |
|
5 |
Examples featuring Minipick, the minimalistic version of Nitpick. |
|
6 |
*) |
|
7 |
||
8 |
header {* Examples Featuring Minipick, the Minimalistic Version of Nitpick *} |
|
9 |
||
10 |
theory Mini_Nits |
|
11 |
imports Main |
|
12 |
begin |
|
13 |
||
14 |
ML {* |
|
15 |
exception FAIL |
|
16 |
||
17 |
(* int -> term -> string *) |
|
35284
9edc2bd6d2bd
enabled Nitpick's support for quotient types + shortened the Nitpick tests a bit
blanchet
parents:
35076
diff
changeset
|
18 |
fun minipick n t = |
9edc2bd6d2bd
enabled Nitpick's support for quotient types + shortened the Nitpick tests a bit
blanchet
parents:
35076
diff
changeset
|
19 |
map (fn k => Minipick.kodkod_problem_from_term @{context} (K k) t) (1 upto n) |
9edc2bd6d2bd
enabled Nitpick's support for quotient types + shortened the Nitpick tests a bit
blanchet
parents:
35076
diff
changeset
|
20 |
|> Minipick.solve_any_kodkod_problem @{theory} |
33197 | 21 |
(* int -> term -> bool *) |
22 |
fun none n t = (minipick n t = "none" orelse raise FAIL) |
|
23 |
fun genuine n t = (minipick n t = "genuine" orelse raise FAIL) |
|
24 |
fun unknown n t = (minipick n t = "unknown" orelse raise FAIL) |
|
25 |
*} |
|
26 |
||
27 |
ML {* genuine 1 @{prop "x = Not"} *} |
|
28 |
ML {* none 1 @{prop "\<exists>x. x = Not"} *} |
|
29 |
ML {* none 1 @{prop "\<not> False"} *} |
|
30 |
ML {* genuine 1 @{prop "\<not> True"} *} |
|
31 |
ML {* none 1 @{prop "\<not> \<not> b \<longleftrightarrow> b"} *} |
|
32 |
ML {* none 1 @{prop True} *} |
|
33 |
ML {* genuine 1 @{prop False} *} |
|
34 |
ML {* genuine 1 @{prop "True \<longleftrightarrow> False"} *} |
|
35 |
ML {* none 1 @{prop "True \<longleftrightarrow> \<not> False"} *} |
|
36 |
ML {* none 5 @{prop "\<forall>x. x = x"} *} |
|
37 |
ML {* none 5 @{prop "\<exists>x. x = x"} *} |
|
38 |
ML {* none 1 @{prop "\<forall>x. x = y"} *} |
|
39 |
ML {* genuine 2 @{prop "\<forall>x. x = y"} *} |
|
40 |
ML {* none 1 @{prop "\<exists>x. x = y"} *} |
|
41 |
ML {* none 2 @{prop "\<exists>x. x = y"} *} |
|
42 |
ML {* none 2 @{prop "\<forall>x\<Colon>'a \<times> 'a. x = x"} *} |
|
43 |
ML {* none 2 @{prop "\<exists>x\<Colon>'a \<times> 'a. x = y"} *} |
|
44 |
ML {* genuine 2 @{prop "\<forall>x\<Colon>'a \<times> 'a. x = y"} *} |
|
45 |
ML {* none 2 @{prop "\<exists>x\<Colon>'a \<times> 'a. x = y"} *} |
|
46 |
ML {* none 1 @{prop "All = Ex"} *} |
|
47 |
ML {* genuine 2 @{prop "All = Ex"} *} |
|
48 |
ML {* none 1 @{prop "All P = Ex P"} *} |
|
49 |
ML {* genuine 2 @{prop "All P = Ex P"} *} |
|
50 |
ML {* none 5 @{prop "x = y \<longrightarrow> P x = P y"} *} |
|
51 |
ML {* none 5 @{prop "(x\<Colon>'a \<times> 'a) = y \<longrightarrow> P x = P y"} *} |
|
52 |
ML {* none 2 @{prop "(x\<Colon>'a \<times> 'a) = y \<longrightarrow> P x y = P y x"} *} |
|
53 |
ML {* none 5 @{prop "\<exists>x\<Colon>'a \<times> 'a. x = y \<longrightarrow> P x = P y"} *} |
|
54 |
ML {* none 2 @{prop "(x\<Colon>'a \<Rightarrow> 'a) = y \<longrightarrow> P x = P y"} *} |
|
55 |
ML {* none 2 @{prop "\<exists>x\<Colon>'a \<Rightarrow> 'a. x = y \<longrightarrow> P x = P y"} *} |
|
56 |
ML {* genuine 1 @{prop "(op =) X = Ex"} *} |
|
57 |
ML {* none 2 @{prop "\<forall>x::'a \<Rightarrow> 'a. x = x"} *} |
|
58 |
ML {* none 1 @{prop "x = y"} *} |
|
59 |
ML {* genuine 1 @{prop "x \<longleftrightarrow> y"} *} |
|
60 |
ML {* genuine 2 @{prop "x = y"} *} |
|
61 |
ML {* genuine 1 @{prop "X \<subseteq> Y"} *} |
|
62 |
ML {* none 1 @{prop "P \<and> Q \<longleftrightarrow> Q \<and> P"} *} |
|
63 |
ML {* none 1 @{prop "P \<and> Q \<longrightarrow> P"} *} |
|
64 |
ML {* none 1 @{prop "P \<or> Q \<longleftrightarrow> Q \<or> P"} *} |
|
65 |
ML {* genuine 1 @{prop "P \<or> Q \<longrightarrow> P"} *} |
|
66 |
ML {* none 1 @{prop "(P \<longrightarrow> Q) \<longleftrightarrow> (\<not> P \<or> Q)"} *} |
|
67 |
ML {* none 5 @{prop "{a} = {a, a}"} *} |
|
68 |
ML {* genuine 2 @{prop "{a} = {a, b}"} *} |
|
69 |
ML {* genuine 1 @{prop "{a} \<noteq> {a, b}"} *} |
|
70 |
ML {* none 5 @{prop "{}\<^sup>+ = {}"} *} |
|
71 |
ML {* none 1 @{prop "{(a, b), (b, c)}\<^sup>+ = {(a, b), (a, c), (b, c)}"} *} |
|
72 |
ML {* genuine 2 @{prop "{(a, b), (b, c)}\<^sup>+ = {(a, b), (a, c), (b, c)}"} *} |
|
73 |
ML {* none 5 @{prop "a \<noteq> c \<Longrightarrow> {(a, b), (b, c)}\<^sup>+ = {(a, b), (a, c), (b, c)}"} *} |
|
74 |
ML {* none 5 @{prop "A \<union> B = (\<lambda>x. A x \<or> B x)"} *} |
|
75 |
ML {* none 5 @{prop "A \<inter> B = (\<lambda>x. A x \<and> B x)"} *} |
|
76 |
ML {* none 5 @{prop "A - B = (\<lambda>x. A x \<and> \<not> B x)"} *} |
|
77 |
ML {* none 5 @{prop "\<exists>a b. (a, b) = (b, a)"} *} |
|
78 |
ML {* genuine 2 @{prop "(a, b) = (b, a)"} *} |
|
79 |
ML {* genuine 2 @{prop "(a, b) \<noteq> (b, a)"} *} |
|
80 |
ML {* none 5 @{prop "\<exists>a b\<Colon>'a \<times> 'a. (a, b) = (b, a)"} *} |
|
81 |
ML {* genuine 2 @{prop "(a\<Colon>'a \<times> 'a, b) = (b, a)"} *} |
|
82 |
ML {* none 5 @{prop "\<exists>a b\<Colon>'a \<times> 'a \<times> 'a. (a, b) = (b, a)"} *} |
|
83 |
ML {* genuine 2 @{prop "(a\<Colon>'a \<times> 'a \<times> 'a, b) \<noteq> (b, a)"} *} |
|
84 |
ML {* none 5 @{prop "\<exists>a b\<Colon>'a \<Rightarrow> 'a. (a, b) = (b, a)"} *} |
|
85 |
ML {* genuine 1 @{prop "(a\<Colon>'a \<Rightarrow> 'a, b) \<noteq> (b, a)"} *} |
|
35284
9edc2bd6d2bd
enabled Nitpick's support for quotient types + shortened the Nitpick tests a bit
blanchet
parents:
35076
diff
changeset
|
86 |
ML {* none 5 @{prop "fst (a, b) = a"} *} |
33197 | 87 |
ML {* none 1 @{prop "fst (a, b) = b"} *} |
88 |
ML {* genuine 2 @{prop "fst (a, b) = b"} *} |
|
89 |
ML {* genuine 2 @{prop "fst (a, b) \<noteq> b"} *} |
|
35284
9edc2bd6d2bd
enabled Nitpick's support for quotient types + shortened the Nitpick tests a bit
blanchet
parents:
35076
diff
changeset
|
90 |
ML {* none 5 @{prop "snd (a, b) = b"} *} |
33197 | 91 |
ML {* none 1 @{prop "snd (a, b) = a"} *} |
92 |
ML {* genuine 2 @{prop "snd (a, b) = a"} *} |
|
93 |
ML {* genuine 2 @{prop "snd (a, b) \<noteq> a"} *} |
|
94 |
ML {* genuine 1 @{prop P} *} |
|
95 |
ML {* genuine 1 @{prop "(\<lambda>x. P) a"} *} |
|
96 |
ML {* genuine 1 @{prop "(\<lambda>x y z. P y x z) a b c"} *} |
|
97 |
ML {* none 5 @{prop "\<exists>f. f = (\<lambda>x. x) \<and> f y = y"} *} |
|
98 |
ML {* genuine 1 @{prop "\<exists>f. f p \<noteq> p \<and> (\<forall>a b. f (a, b) = (a, b))"} *} |
|
99 |
ML {* none 2 @{prop "\<exists>f. \<forall>a b. f (a, b) = (a, b)"} *} |
|
100 |
ML {* none 3 @{prop "f = (\<lambda>a b. (b, a)) \<longrightarrow> f x y = (y, x)"} *} |
|
101 |
ML {* genuine 2 @{prop "f = (\<lambda>a b. (b, a)) \<longrightarrow> f x y = (x, y)"} *} |
|
102 |
||
103 |
end |