src/HOLCF/IOA/meta_theory/TrivEx2.thy
author wenzelm
Sun, 25 Oct 1998 12:33:27 +0100
changeset 5769 6a422b22ba02
parent 4816 64f075872f69
permissions -rw-r--r--
tuned checklist;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
4559
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     1
(*  Title:      HOLCF/IOA/TrivEx.thy
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     2
    ID:         $Id$
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     3
    Author:     Olaf Mueller
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     4
    Copyright   1995  TU Muenchen
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     5
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     6
Trivial Abstraction Example with fairness
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     7
*)
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     8
4816
64f075872f69 simplification of explicit theory usage and merges
oheimb
parents: 4559
diff changeset
     9
TrivEx2 = Abstraction + IOA +
4559
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    10
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    11
datatype action = INC
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    12
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    13
consts
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    14
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    15
C_asig   ::  action signature
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    16
C_trans  :: (action, nat)transition set
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    17
C_ioa    :: (action, nat)ioa
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    18
C_live_ioa :: (action, nat)live_ioa
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    19
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    20
A_asig   :: action signature
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    21
A_trans  :: (action, bool)transition set
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    22
A_ioa    :: (action, bool)ioa
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    23
A_live_ioa :: (action, bool)live_ioa
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    24
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    25
h_abs    :: "nat => bool"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    26
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    27
defs
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    28
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    29
C_asig_def
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    30
  "C_asig == ({},{INC},{})"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    31
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    32
C_trans_def "C_trans ==                                           
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    33
 {tr. let s = fst(tr);                                               
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    34
          t = snd(snd(tr))                                           
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    35
      in case fst(snd(tr))                                           
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    36
      of                                                             
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    37
      INC       => t = Suc(s)}"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    38
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    39
C_ioa_def "C_ioa == 
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    40
 (C_asig, {0}, C_trans,{},{})"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    41
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    42
C_live_ioa_def 
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    43
  "C_live_ioa == (C_ioa, WF C_ioa {INC})"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    44
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    45
A_asig_def
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    46
  "A_asig == ({},{INC},{})"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    47
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    48
A_trans_def "A_trans ==                                           
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    49
 {tr. let s = fst(tr);                                               
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    50
          t = snd(snd(tr))                                           
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    51
      in case fst(snd(tr))                                           
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    52
      of                                                             
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    53
      INC       => t = True}"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    54
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    55
A_ioa_def "A_ioa == 
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    56
 (A_asig, {False}, A_trans,{},{})"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    57
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    58
A_live_ioa_def 
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    59
  "A_live_ioa == (A_ioa, WF A_ioa {INC})"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    60
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    61
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    62
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    63
h_abs_def
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    64
  "h_abs n == n~=0"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    65
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    66
rules
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    67
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    68
MC_result
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    69
  "validLIOA (A_ioa,WF A_ioa {INC}) (<>[] <%(b,a,c). b>)"
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    70
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    71
end