diff -r 722bf1319be5 -r fd1be45b64bf IOA/meta_theory/Solve.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/IOA/meta_theory/Solve.thy Wed Nov 02 11:50:09 1994 +0100 @@ -0,0 +1,20 @@ +(* Methods of proof for IOA. *) + +Solve = IOA + + +consts + + is_weak_pmap :: "['c => 'a, ('action,'c)ioa,('action,'a)ioa] => bool" + +rules + +is_weak_pmap_def + "is_weak_pmap(f,C,A) == \ +\ (!s:starts_of(C). f(s):starts_of(A)) & \ +\ (!s t a. reachable(C,s) & \ +\ :trans_of(C) \ +\ --> if(a:externals(asig_of(C)), \ +\ :trans_of(A), \ +\ f(s)=f(t)))" + +end