src/HOL/HOLCF/IOA/Abstraction.thy
changeset 62441 e5e38e1f2dd4
parent 62195 799a5306e2ed
child 63549 b0d31c7def86
--- a/src/HOL/HOLCF/IOA/Abstraction.thy	Sat Feb 27 21:04:13 2016 +0100
+++ b/src/HOL/HOLCF/IOA/Abstraction.thy	Sat Feb 27 21:09:43 2016 +0100
@@ -53,7 +53,7 @@
 
 (* analog to the proved thm strength_Next - proof skipped as trivial *)
 axiomatization where
-  weak_Next: "temp_weakening P Q h \<Longrightarrow> temp_weakening (Next P) (Next Q) h"
+  weak_Next: "temp_weakening P Q h \<Longrightarrow> temp_weakening (\<circle>P) (\<circle>Q) h"
 
 
 subsection \<open>\<open>cex_abs\<close>\<close>
@@ -382,7 +382,7 @@
   apply (pair a)
   done
 
-lemma strength_Next: "temp_strengthening P Q h \<Longrightarrow> temp_strengthening (Next P) (Next Q) h"
+lemma strength_Next: "temp_strengthening P Q h \<Longrightarrow> temp_strengthening (\<circle>P) (\<circle>Q) h"
   apply (unfold temp_strengthening_def state_strengthening_def temp_sat_def satisfies_def Next_def)
   apply simp
   apply auto