# HG changeset patch # User wenzelm # Date 1446679033 -3600 # Node ID c49a8ebd30ccc946a9a3630e0ac847a34fbc8a21 # Parent 634cd44bb1d3dd13baae8beb239c3143e1556c61 isabelle update_cartouches -c; diff -r 634cd44bb1d3 -r c49a8ebd30cc src/Doc/Eisbach/Manual.thy --- a/src/Doc/Eisbach/Manual.thy Thu Nov 05 00:02:30 2015 +0100 +++ b/src/Doc/Eisbach/Manual.thy Thu Nov 05 00:17:13 2015 +0100 @@ -249,16 +249,16 @@ \ lemmas [intros] = - conjI -- \@{thm conjI}\ - impI -- \@{thm impI}\ - disjCI -- \@{thm disjCI}\ - iffI -- \@{thm iffI}\ - notI -- \@{thm notI}\ + conjI \ \@{thm conjI}\ + impI \ \@{thm impI}\ + disjCI \ \@{thm disjCI}\ + iffI \ \@{thm iffI}\ + notI \ \@{thm notI}\ lemmas [elims] = - impCE -- \@{thm impCE}\ - conjE -- \@{thm conjE}\ - disjE -- \@{thm disjE}\ + impCE \ \@{thm impCE}\ + conjE \ \@{thm conjE}\ + disjE \ \@{thm disjE}\ lemma "(A \ B) \ (A \ C) \ (B \ C) \ C" by prop_solver diff -r 634cd44bb1d3 -r c49a8ebd30cc src/Doc/Implementation/ML.thy --- a/src/Doc/Implementation/ML.thy Thu Nov 05 00:02:30 2015 +0100 +++ b/src/Doc/Implementation/ML.thy Thu Nov 05 00:17:13 2015 +0100 @@ -578,7 +578,7 @@ ML_prf %"ML" \val a = 1\ { ML_prf %"ML" \val b = a + 1\ - } -- \Isar block structure ignored by ML environment\ + } \ \Isar block structure ignored by ML environment\ ML_prf %"ML" \val c = b + 1\ end diff -r 634cd44bb1d3 -r c49a8ebd30cc src/Doc/Implementation/Prelim.thy --- a/src/Doc/Implementation/Prelim.thy Thu Nov 05 00:02:30 2015 +0100 +++ b/src/Doc/Implementation/Prelim.thy Thu Nov 05 00:17:13 2015 +0100 @@ -471,17 +471,17 @@ begin declare [[show_types = false]] - -- \declaration within (local) theory context\ + \ \declaration within (local) theory context\ notepad begin note [[show_types = true]] - -- \declaration within proof (forward mode)\ + \ \declaration within proof (forward mode)\ term x have "x = x" using [[show_types = false]] - -- \declaration within proof (backward mode)\ + \ \declaration within proof (backward mode)\ .. end diff -r 634cd44bb1d3 -r c49a8ebd30cc src/Doc/Implementation/Proof.thy --- a/src/Doc/Implementation/Proof.thy Thu Nov 05 00:02:30 2015 +0100 +++ b/src/Doc/Implementation/Proof.thy Thu Nov 05 00:17:13 2015 +0100 @@ -58,14 +58,14 @@ notepad begin { - fix x -- \all potential occurrences of some \x::\\ are fixed\ + fix x \ \all potential occurrences of some \x::\\ are fixed\ { - have "x::'a \ x" -- \implicit type assignment by concrete occurrence\ + have "x::'a \ x" \ \implicit type assignment by concrete occurrence\ by (rule reflexive) } - thm this -- \result still with fixed type \'a\\ + thm this \ \result still with fixed type \'a\\ } - thm this -- \fully general result for arbitrary \?x::?'a\\ + thm this \ \fully general result for arbitrary \?x::?'a\\ end text \The Isabelle/Isar proof context manages the details of term diff -r 634cd44bb1d3 -r c49a8ebd30cc src/Doc/Isar_Ref/First_Order_Logic.thy --- a/src/Doc/Isar_Ref/First_Order_Logic.thy Thu Nov 05 00:02:30 2015 +0100 +++ b/src/Doc/Isar_Ref/First_Order_Logic.thy Thu Nov 05 00:17:13 2015 +0100 @@ -357,10 +357,10 @@ theorem assumes "\x. \y. R x y" shows "\y. \x. R x y" -proof -- \\\\ introduction\ - obtain x where "\y. R x y" using \\x. \y. R x y\ .. -- \\\\ elimination\ - fix y have "R x y" using \\y. R x y\ .. -- \\\\ destruction\ - then show "\x. R x y" .. -- \\\\ introduction\ +proof \ \\\\ introduction\ + obtain x where "\y. R x y" using \\x. \y. R x y\ .. \ \\\\ elimination\ + fix y have "R x y" using \\y. R x y\ .. \ \\\\ destruction\ + then show "\x. R x y" .. \ \\\\ introduction\ qed diff -r 634cd44bb1d3 -r c49a8ebd30cc src/Doc/Isar_Ref/Synopsis.thy --- a/src/Doc/Isar_Ref/Synopsis.thy Thu Nov 05 00:02:30 2015 +0100 +++ b/src/Doc/Isar_Ref/Synopsis.thy Thu Nov 05 00:17:13 2015 +0100 @@ -17,11 +17,11 @@ notepad begin txt \Locally fixed entities:\ - fix x -- \local constant, without any type information yet\ - fix x :: 'a -- \variant with explicit type-constraint for subsequent use\ + fix x \ \local constant, without any type information yet\ + fix x :: 'a \ \variant with explicit type-constraint for subsequent use\ fix a b - assume "a = b" -- \type assignment at first occurrence in concrete term\ + assume "a = b" \ \type assignment at first occurrence in concrete term\ txt \Definitions (non-polymorphic):\ def x \ "t::'a" @@ -234,7 +234,7 @@ proof - term ?thesis show ?thesis sorry - term ?thesis -- \static!\ + term ?thesis \ \static!\ qed term "\" thm this @@ -345,7 +345,7 @@ moreover { assume C have R sorry } ultimately - have R by blast -- \``big-bang integration'' of proof blocks (occasionally fragile)\ + have R by blast \ \``big-bang integration'' of proof blocks (occasionally fragile)\ end @@ -364,7 +364,7 @@ begin fix n :: nat have "P n" - proof (rule nat.induct) -- \fragile rule application!\ + proof (rule nat.induct) \ \fragile rule application!\ show "P 0" sorry next fix n :: nat @@ -503,7 +503,7 @@ from \A x 0\ show "Q x 0" sorry next case (Suc n) - from \\x. A x n \ Q x n\ -- \arbitrary instances can be produced here\ + from \\x. A x n \ Q x n\ \ \arbitrary instances can be produced here\ and \A x (Suc n)\ show "Q x (Suc n)" sorry qed end @@ -675,9 +675,9 @@ begin assume a: A and b: B thm conjI - thm conjI [of A B] -- "instantiation" - thm conjI [of A B, OF a b] -- "instantiation and composition" - thm conjI [OF a b] -- "composition via unification (trivial)" + thm conjI [of A B] \ "instantiation" + thm conjI [of A B, OF a b] \ "instantiation and composition" + thm conjI [OF a b] \ "composition via unification (trivial)" thm conjI [OF \A\ \B\] thm conjI [OF disjI1] @@ -710,9 +710,9 @@ fix x assume "A x" show "B x" sorry - } -- "implicit block structure made explicit" + } \ "implicit block structure made explicit" note \\x. A x \ B x\ - -- "side exit for the resulting rule" + \ "side exit for the resulting rule" qed end @@ -726,12 +726,12 @@ notepad begin - assume r1: "A \ B \ C" -- \simple rule (Horn clause)\ + assume r1: "A \ B \ C" \ \simple rule (Horn clause)\ - have A sorry -- "prefix of facts via outer sub-proof" + have A sorry \ "prefix of facts via outer sub-proof" then have C proof (rule r1) - show B sorry -- "remaining rule premises via inner sub-proof" + show B sorry \ "remaining rule premises via inner sub-proof" qed have C @@ -750,7 +750,7 @@ next - assume r2: "A \ (\x. B1 x \ B2 x) \ C" -- \nested rule\ + assume r2: "A \ (\x. B1 x \ B2 x) \ C" \ \nested rule\ have A sorry then have C @@ -850,31 +850,31 @@ notepad begin have "A \ B" - proof -- \two strictly isolated subproofs\ + proof \ \two strictly isolated subproofs\ show A sorry next show B sorry qed have "A \ B" - proof -- \one simultaneous sub-proof\ + proof \ \one simultaneous sub-proof\ show A and B sorry qed have "A \ B" - proof -- \two subproofs in the same context\ + proof \ \two subproofs in the same context\ show A sorry show B sorry qed have "A \ B" - proof -- \swapped order\ + proof \ \swapped order\ show B sorry show A sorry qed have "A \ B" - proof -- \sequential subproofs\ + proof \ \sequential subproofs\ show A sorry show B using \A\ sorry qed @@ -941,9 +941,9 @@ following typical representatives: \ -thm exE -- \local parameter\ -thm conjE -- \local premises\ -thm disjE -- \split into cases\ +thm exE \ \local parameter\ +thm conjE \ \local premises\ +thm disjE \ \split into cases\ text \ Combining these characteristics leads to the following general scheme @@ -1001,7 +1001,7 @@ print_statement disjE lemma - assumes A1 and A2 -- \assumptions\ + assumes A1 and A2 \ \assumptions\ obtains (case1) x y where "B1 x y" and "C1 x y" | (case2) x y where "B2 x y" and "C2 x y"