author | blanchet |
Tue, 14 Sep 2010 13:24:18 +0200 | |
changeset 39359 | 6f49c7fbb1b1 |
parent 32689 | 860e1a2317bd |
child 42767 | e6d920bea7a6 |
permissions | -rw-r--r-- |
13786 | 1 |
(* Title: HOL/UNITY/UNITY_Main.thy |
2 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
3 |
Copyright 2003 University of Cambridge |
|
13798 | 4 |
*) |
13786 | 5 |
|
13798 | 6 |
header{*Comprehensive UNITY Theory*} |
13786 | 7 |
|
32689 | 8 |
theory UNITY_Main |
9 |
imports Detects PPROD Follows ProgressSets |
|
10 |
uses "UNITY_tactics.ML" |
|
11 |
begin |
|
13786 | 12 |
|
16184
80617b8d33c5
renamed "constrains" to "safety" to avoid keyword clash
paulson
parents:
15032
diff
changeset
|
13 |
method_setup safety = {* |
30549 | 14 |
Scan.succeed (fn ctxt => |
32149
ef59550a55d3
renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;
wenzelm
parents:
30549
diff
changeset
|
15 |
SIMPLE_METHOD' (constrains_tac (clasimpset_of ctxt))) *} |
13786 | 16 |
"for proving safety properties" |
17 |
||
18 |
method_setup ensures_tac = {* |
|
30549 | 19 |
Args.goal_spec -- Scan.lift Args.name_source >> |
32149
ef59550a55d3
renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;
wenzelm
parents:
30549
diff
changeset
|
20 |
(fn (quant, s) => fn ctxt => SIMPLE_METHOD'' quant (ensures_tac (clasimpset_of ctxt) s)) |
30549 | 21 |
*} "for proving progress properties" |
13786 | 22 |
|
23 |
end |