src/HOL/IOA/Solve.thy
changeset 3078 984866a8f905
child 4530 ac1821645636
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/IOA/Solve.thy	Wed Apr 30 11:56:17 1997 +0200
@@ -0,0 +1,22 @@
+(*  Title:      HOL/IOA/meta_theory/Solve.thy
+    ID:         $Id$
+    Author:     Tobias Nipkow & Konrad Slind
+    Copyright   1994  TU Muenchen
+
+Weak possibilities mapping (abstraction)
+*)
+
+Solve = IOA +
+
+constdefs
+
+  is_weak_pmap :: "['c => 'a, ('action,'c)ioa,('action,'a)ioa] => bool"
+  "is_weak_pmap f C A ==                          
+   (!s:starts_of(C). f(s):starts_of(A)) &        
+   (!s t a. reachable C s &                      
+            (s,a,t):trans_of(C)                  
+            --> (if a:externals(asig_of(C)) then 
+                   (f(s),a,f(t)):trans_of(A)     
+                 else f(s)=f(t)))"
+
+end