src/HOL/IOA/meta_theory/Solve.thy
changeset 972 e61b058d58d2
parent 966 3fd66f245ad7
child 1151 c820b3cc3df0
equal deleted inserted replaced
971:f4815812665b 972:e61b058d58d2
    16 
    16 
    17 is_weak_pmap_def
    17 is_weak_pmap_def
    18   "is_weak_pmap f C A ==                          \
    18   "is_weak_pmap f C A ==                          \
    19 \   (!s:starts_of(C). f(s):starts_of(A)) &        \
    19 \   (!s:starts_of(C). f(s):starts_of(A)) &        \
    20 \   (!s t a. reachable C s &                      \
    20 \   (!s t a. reachable C s &                      \
    21 \            <s,a,t>:trans_of(C)                  \
    21 \            (s,a,t):trans_of(C)                  \
    22 \            --> (if a:externals(asig_of(C)) then \
    22 \            --> (if a:externals(asig_of(C)) then \
    23 \                   <f(s),a,f(t)>:trans_of(A)     \
    23 \                   (f(s),a,f(t)):trans_of(A)     \
    24 \                 else f(s)=f(t)))"
    24 \                 else f(s)=f(t)))"
    25 
    25 
    26 end
    26 end