diff -r 703edebd1d92 -r f1ecba0272f9 src/HOL/UNITY/Comp/Progress.thy --- a/src/HOL/UNITY/Comp/Progress.thy Wed May 25 11:49:40 2016 +0200 +++ b/src/HOL/UNITY/Comp/Progress.thy Wed May 25 11:50:58 2016 +0200 @@ -5,12 +5,12 @@ David Meier's thesis *) -section{*Progress Set Examples*} +section\Progress Set Examples\ theory Progress imports "../UNITY_Main" begin -subsection {*The Composition of Two Single-Assignment Programs*} -text{*Thesis Section 4.4.2*} +subsection \The Composition of Two Single-Assignment Programs\ +text\Thesis Section 4.4.2\ definition FF :: "int program" where "FF = mk_total_program (UNIV, {range (\x. (x, x+1))}, UNIV)" @@ -18,7 +18,7 @@ definition GG :: "int program" where "GG = mk_total_program (UNIV, {range (\x. (x, 2*x))}, UNIV)" -subsubsection {*Calculating @{term "wens_set FF (atLeast k)"}*} +subsubsection \Calculating @{term "wens_set FF (atLeast k)"}\ lemma Domain_actFF: "Domain (range (\x::int. (x, x + 1))) = UNIV" by force @@ -62,7 +62,7 @@ apply (simp add: wens_single_finite_FF) done -subsubsection {*Proving @{term "FF \ UNIV leadsTo atLeast (k::int)"}*} +subsubsection \Proving @{term "FF \ UNIV leadsTo atLeast (k::int)"}\ lemma atLeast_ensures: "FF \ atLeast (k - 1) ensures atLeast (k::int)" apply (simp add: Progress.wens_FF [symmetric] wens_ensures) @@ -86,7 +86,7 @@ apply (rule leadsTo_UN [OF atLeast_leadsTo]) done -text{*Result (4.39): Applying the leadsTo-Join Theorem*} +text\Result (4.39): Applying the leadsTo-Join Theorem\ theorem "FF\GG \ atLeast 0 leadsTo atLeast (k::int)" apply (subgoal_tac "FF\GG \ (atLeast 0 \ atLeast 0) leadsTo atLeast k") apply simp