# HG changeset patch # User wenzelm # Date 1456603783 -3600 # Node ID e5e38e1f2dd4c844abe86051b5954fd6d942e064 # Parent 31fa592761da3fae04e8fc6955797bf1a0c139ca more symbols; diff -r 31fa592761da -r e5e38e1f2dd4 src/HOL/HOLCF/IOA/Abstraction.thy --- 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 \ temp_weakening (Next P) (Next Q) h" + weak_Next: "temp_weakening P Q h \ temp_weakening (\P) (\Q) h" subsection \\cex_abs\\ @@ -382,7 +382,7 @@ apply (pair a) done -lemma strength_Next: "temp_strengthening P Q h \ temp_strengthening (Next P) (Next Q) h" +lemma strength_Next: "temp_strengthening P Q h \ temp_strengthening (\P) (\Q) h" apply (unfold temp_strengthening_def state_strengthening_def temp_sat_def satisfies_def Next_def) apply simp apply auto diff -r 31fa592761da -r e5e38e1f2dd4 src/HOL/HOLCF/IOA/TL.thy --- a/src/HOL/HOLCF/IOA/TL.thy Sat Feb 27 21:04:13 2016 +0100 +++ b/src/HOL/HOLCF/IOA/TL.thy Sat Feb 27 21:09:43 2016 +0100 @@ -22,8 +22,8 @@ where "Init P s = P (unlift (HD $ s))" \ \this means that for \nil\ and \UU\ the effect is unpredictable\ -definition Next :: "'a temporal \ 'a temporal" - where "(Next P) s \ (if TL $ s = UU \ TL $ s = nil then P s else P (TL $ s))" +definition Next :: "'a temporal \ 'a temporal" ("\(_)" [80] 80) + where "(\P) s \ (if TL $ s = UU \ TL $ s = nil then P s else P (TL $ s))" definition suffix :: "'a Seq \ 'a Seq \ bool" where "suffix s2 s \ (\s1. Finite s1 \ s = s1 @@ s2)" @@ -120,14 +120,14 @@ lemmas tsuffix_TL2 = conjI [THEN tsuffix_TL] -lemma LTL1: "s \ UU \ s \ nil \ (s \ \F \<^bold>\ (F \<^bold>\ (Next (\F))))" +lemma LTL1: "s \ UU \ s \ nil \ (s \ \F \<^bold>\ (F \<^bold>\ (\(\F))))" supply if_split [split del] apply (unfold Next_def satisfies_def NOT_def IMPLIES_def AND_def Box_def) apply auto text \\\F \<^bold>\ F\\ apply (erule_tac x = "s" in allE) apply (simp add: tsuffix_def suffix_refl) - text \\\F \<^bold>\ Next \F\\ + text \\\F \<^bold>\ \\F\\ apply (simp split add: if_split) apply auto apply (drule tsuffix_TL2) @@ -135,13 +135,13 @@ apply auto done -lemma LTL2a: "s \ \<^bold>\ (Next F) \<^bold>\ (Next (\<^bold>\ F))" +lemma LTL2a: "s \ \<^bold>\ (\F) \<^bold>\ (\(\<^bold>\ F))" by (simp add: Next_def satisfies_def NOT_def IMPLIES_def) -lemma LTL2b: "s \ (Next (\<^bold>\ F)) \<^bold>\ (\<^bold>\ (Next F))" +lemma LTL2b: "s \ (\(\<^bold>\ F)) \<^bold>\ (\<^bold>\ (\F))" by (simp add: Next_def satisfies_def NOT_def IMPLIES_def) -lemma LTL3: "ex \ (Next (F \<^bold>\ G)) \<^bold>\ (Next F) \<^bold>\ (Next G)" +lemma LTL3: "ex \ (\(F \<^bold>\ G)) \<^bold>\ (\F) \<^bold>\ (\G)" by (simp add: Next_def satisfies_def NOT_def IMPLIES_def) lemma ModusPonens: "\<^bold>\ (P \<^bold>\ Q) \ \<^bold>\ P \ \<^bold>\ Q" diff -r 31fa592761da -r e5e38e1f2dd4 src/HOL/HOLCF/IOA/TLS.thy --- a/src/HOL/HOLCF/IOA/TLS.thy Sat Feb 27 21:04:13 2016 +0100 +++ b/src/HOL/HOLCF/IOA/TLS.thy Sat Feb 27 21:09:43 2016 +0100 @@ -137,7 +137,7 @@ lemma TL_TLS: "\s a t. (P s) \ s \a\A\ t \ (Q t) \ ex \ (Init (\(s, a, t). P s) \<^bold>\ Init (\(s, a, t). s \a\A\ t) - \<^bold>\ (Next (Init (\(s, a, t). Q s))))" + \<^bold>\ (\(Init (\(s, a, t). Q s))))" apply (unfold Init_def Next_def temp_sat_def satisfies_def IMPLIES_def AND_def) apply clarify apply (simp split add: if_split)