| author | wenzelm |
| Mon, 02 Jan 2006 20:50:17 +0100 | |
| changeset 18539 | 35b9ed76b59a |
| parent 17233 | 41eee2e7b465 |
| child 19741 | f65265d71426 |
| permissions | -rw-r--r-- |
| 4559 | 1 |
(* Title: HOLCF/IOA/meta_theory/TLS.thy |
2 |
ID: $Id$ |
|
| 12218 | 3 |
Author: Olaf Müller |
| 17233 | 4 |
*) |
| 4559 | 5 |
|
| 17233 | 6 |
header {* A General Temporal Logic *}
|
| 4559 | 7 |
|
| 17233 | 8 |
theory TL |
9 |
imports Pred Sequence |
|
10 |
begin |
|
11 |
||
12 |
defaultsort type |
|
| 4559 | 13 |
|
14 |
types |
|
| 17233 | 15 |
'a temporal = "'a Seq predicate" |
| 4559 | 16 |
|
17 |
||
| 17233 | 18 |
consts |
| 4559 | 19 |
suffix :: "'a Seq => 'a Seq => bool" |
20 |
tsuffix :: "'a Seq => 'a Seq => bool" |
|
21 |
||
22 |
validT :: "'a Seq predicate => bool" |
|
23 |
||
24 |
unlift :: "'a lift => 'a" |
|
25 |
||
26 |
Init ::"'a predicate => 'a temporal" ("<_>" [0] 1000)
|
|
27 |
||
28 |
Box ::"'a temporal => 'a temporal" ("[] (_)" [80] 80)
|
|
29 |
Diamond ::"'a temporal => 'a temporal" ("<> (_)" [80] 80)
|
|
| 17233 | 30 |
Next ::"'a temporal => 'a temporal" |
| 4559 | 31 |
Leadsto ::"'a temporal => 'a temporal => 'a temporal" (infixr "~>" 22) |
32 |
||
|
12114
a8e860c86252
eliminated old "symbols" syntax, use "xsymbols" instead;
wenzelm
parents:
12028
diff
changeset
|
33 |
syntax (xsymbols) |
| 17233 | 34 |
"Box" ::"'a temporal => 'a temporal" ("\<box> (_)" [80] 80)
|
35 |
"Diamond" ::"'a temporal => 'a temporal" ("\<diamond> (_)" [80] 80)
|
|
36 |
"Leadsto" ::"'a temporal => 'a temporal => 'a temporal" (infixr "\<leadsto>" 22) |
|
37 |
||
| 4559 | 38 |
defs |
39 |
||
| 17233 | 40 |
unlift_def: |
41 |
"unlift x == (case x of |
|
| 12028 | 42 |
UU => arbitrary |
| 4559 | 43 |
| Def y => y)" |
44 |
||
45 |
(* this means that for nil and UU the effect is unpredictable *) |
|
| 17233 | 46 |
Init_def: |
47 |
"Init P s == (P (unlift (HD$s)))" |
|
| 4559 | 48 |
|
| 17233 | 49 |
suffix_def: |
50 |
"suffix s2 s == ? s1. (Finite s1 & s = s1 @@ s2)" |
|
| 4559 | 51 |
|
| 17233 | 52 |
tsuffix_def: |
| 4559 | 53 |
"tsuffix s2 s == s2 ~= nil & s2 ~= UU & suffix s2 s" |
54 |
||
| 17233 | 55 |
Box_def: |
| 4559 | 56 |
"([] P) s == ! s2. tsuffix s2 s --> P s2" |
57 |
||
| 17233 | 58 |
Next_def: |
| 10835 | 59 |
"(Next P) s == if (TL$s=UU | TL$s=nil) then (P s) else P (TL$s)" |
| 4559 | 60 |
|
| 17233 | 61 |
Diamond_def: |
| 4559 | 62 |
"<> P == .~ ([] (.~ P))" |
63 |
||
| 17233 | 64 |
Leadsto_def: |
65 |
"P ~> Q == ([] (P .--> (<> Q)))" |
|
| 4559 | 66 |
|
| 17233 | 67 |
validT_def: |
| 4559 | 68 |
"validT P == ! s. s~=UU & s~=nil --> (s |= P)" |
69 |
||
| 17233 | 70 |
ML {* use_legacy_bindings (the_context ()) *}
|
71 |
||
72 |
end |