diff -r 0242c9c980df -r a31203f58b20 doc-src/IsarRef/Thy/Quick_Reference.thy --- a/doc-src/IsarRef/Thy/Quick_Reference.thy Thu May 08 14:52:07 2008 +0200 +++ b/doc-src/IsarRef/Thy/Quick_Reference.thy Thu May 08 22:05:15 2008 +0200 @@ -20,65 +20,78 @@ @{command "using"}~@{text a} & indicate use of additional facts \\ @{command "unfolding"}~@{text a} & unfold definitional equations \\ @{command "proof"}~@{text "m\<^sub>1"}~\dots~@{command "qed"}~@{text "m\<^sub>2"} & indicate proof structure and refinements \\ - @{command "{"}~\dots~@{command "}"} & indicate explicit blocks \\ + @{command "{"}~@{text "\"}~@{command "}"} & indicate explicit blocks \\ @{command "next"} & switch blocks \\ @{command "note"}~@{text "a = b"} & reconsider facts \\ @{command "let"}~@{text "p = t"} & abbreviate terms by higher-order matching \\ \end{tabular} - \begin{matharray}{rcl} - @{text "theory\stmt"} & = & @{command "theorem"}~@{text "name: props proof"} \Or @{command "definition"}~\dots \Or \dots \\[1ex] + \medskip + + \begin{tabular}{rcl} + @{text "theory\stmt"} & = & @{command "theorem"}~@{text "name: props proof |"}~~@{command "definition"}~@{text "\ | \"} \\[1ex] @{text "proof"} & = & @{text "prfx\<^sup>*"}~@{command "proof"}~@{text "method stmt\<^sup>*"}~@{command "qed"}~@{text method} \\ - & \Or & @{text "prfx\<^sup>*"}~@{command "done"} \\[1ex] + & @{text "|"} & @{text "prfx\<^sup>*"}~@{command "done"} \\[1ex] @{text prfx} & = & @{command "apply"}~@{text method} \\ - & \Or & @{command "using"}~@{text "facts"} \\ - & \Or & @{command "unfolding"}~@{text "facts"} \\ + & @{text "|"} & @{command "using"}~@{text "facts"} \\ + & @{text "|"} & @{command "unfolding"}~@{text "facts"} \\ @{text stmt} & = & @{command "{"}~@{text "stmt\<^sup>*"}~@{command "}"} \\ - & \Or & @{command "next"} \\ - & \Or & @{command "note"}~@{text "name = facts"} \\ - & \Or & @{command "let"}~@{text "term = term"} \\ - & \Or & @{command "fix"}~@{text "var\<^sup>+"} \\ - & \Or & @{command "assume"}~@{text "name: props"} \\ - & \Or & @{command "then"}@{text "\<^sup>?"}~@{text goal} \\ + & @{text "|"} & @{command "next"} \\ + & @{text "|"} & @{command "note"}~@{text "name = facts"} \\ + & @{text "|"} & @{command "let"}~@{text "term = term"} \\ + & @{text "|"} & @{command "fix"}~@{text "var\<^sup>+"} \\ + & @{text "|"} & @{command "assume"}~@{text "name: props"} \\ + & @{text "|"} & @{command "then"}@{text "\<^sup>?"}~@{text goal} \\ @{text goal} & = & @{command "have"}~@{text "name: props proof"} \\ - & \Or & @{command "show"}~@{text "name: props proof"} \\ - \end{matharray} + & @{text "|"} & @{command "show"}~@{text "name: props proof"} \\ + \end{tabular} *} subsection {* Abbreviations and synonyms *} text {* - \begin{matharray}{rcl} - @{command "by"}~@{text "m\<^sub>1 m\<^sub>2"} & \equiv & @{command "proof"}~@{text "m\<^sub>1"}~@{command "qed"}~@{text "m\<^sub>2"} \\ - @{command ".."} & \equiv & @{command "by"}~@{text rule} \\ - @{command "."} & \equiv & @{command "by"}~@{text this} \\ - @{command "hence"} & \equiv & @{command "then"}~@{command "have"} \\ - @{command "thus"} & \equiv & @{command "then"}~@{command "show"} \\ - @{command "from"}~@{text a} & \equiv & @{command "note"}~@{text a}~@{command "then"} \\ - @{command "with"}~@{text a} & \equiv & @{command "from"}~@{text "a \ this"} \\[1ex] - @{command "from"}~@{text this} & \equiv & @{command "then"} \\ - @{command "from"}~@{text this}~@{command "have"} & \equiv & @{command "hence"} \\ - @{command "from"}~@{text this}~@{command "show"} & \equiv & @{command "thus"} \\ - \end{matharray} + \begin{tabular}{rcl} + @{command "by"}~@{text "m\<^sub>1 m\<^sub>2"} & @{text "\"} & + @{command "proof"}~@{text "m\<^sub>1"}~@{command "qed"}~@{text "m\<^sub>2"} \\ + @{command ".."} & @{text "\"} & @{command "by"}~@{text rule} \\ + @{command "."} & @{text "\"} & @{command "by"}~@{text this} \\ + @{command "hence"} & @{text "\"} & @{command "then"}~@{command "have"} \\ + @{command "thus"} & @{text "\"} & @{command "then"}~@{command "show"} \\ + @{command "from"}~@{text a} & @{text "\"} & @{command "note"}~@{text a}~@{command "then"} \\ + @{command "with"}~@{text a} & @{text "\"} & @{command "from"}~@{text "a \ this"} \\[1ex] + @{command "from"}~@{text this} & @{text "\"} & @{command "then"} \\ + @{command "from"}~@{text this}~@{command "have"} & @{text "\"} & @{command "hence"} \\ + @{command "from"}~@{text this}~@{command "show"} & @{text "\"} & @{command "thus"} \\ + \end{tabular} *} subsection {* Derived elements *} text {* - \begin{matharray}{rcl} - @{command "also"}@{text "\<^sub>0"} & \approx & @{command "note"}~@{text "calculation = this"} \\ - @{command "also"}@{text "\<^sub>n\<^sub>+\<^sub>1"} & \approx & @{command "note"}~@{text "calculation = trans [OF calculation this]"} \\ - @{command "finally"} & \approx & @{command "also"}~@{command "from"}~@{text calculation} \\[0.5ex] - @{command "moreover"} & \approx & @{command "note"}~@{text "calculation = calculation this"} \\ - @{command "ultimately"} & \approx & @{command "moreover"}~@{command "from"}~@{text calculation} \\[0.5ex] - @{command "presume"}~@{text "a: \"} & \approx & @{command "assume"}~@{text "a: \"} \\ - @{command "def"}~@{text "a: x \ t"} & \approx & @{command "fix"}~@{text x}~@{command "assume"}~@{text "a: x \ t"} \\ - @{command "obtain"}~@{text "x \ a: \"} & \approx & \dots~@{command "fix"}~@{text x}~@{command "assume"}~@{text "a: \"} \\ - @{command "case"}~@{text c} & \approx & @{command "fix"}~@{text x}~@{command "assume"}~@{text "c: \"} \\ - @{command "sorry"} & \approx & @{command "by"}~@{text cheating} \\ - \end{matharray} + \begin{tabular}{rcl} + @{command "also"}@{text "\<^sub>0"} & @{text "\"} & + @{command "note"}~@{text "calculation = this"} \\ + @{command "also"}@{text "\<^sub>n\<^sub>+\<^sub>1"} & @{text "\"} & + @{command "note"}~@{text "calculation = trans [OF calculation this]"} \\ + @{command "finally"} & @{text "\"} & + @{command "also"}~@{command "from"}~@{text calculation} \\[0.5ex] + @{command "moreover"} & @{text "\"} & + @{command "note"}~@{text "calculation = calculation this"} \\ + @{command "ultimately"} & @{text "\"} & + @{command "moreover"}~@{command "from"}~@{text calculation} \\[0.5ex] + @{command "presume"}~@{text "a: \"} & @{text "\"} & + @{command "assume"}~@{text "a: \"} \\ + @{command "def"}~@{text "a: x \ t"} & @{text "\"} & + @{command "fix"}~@{text x}~@{command "assume"}~@{text "a: x \ t"} \\ + @{command "obtain"}~@{text "x \ a: \"} & @{text "\"} & + @{text "\"}~@{command "fix"}~@{text x}~@{command "assume"}~@{text "a: \"} \\ + @{command "case"}~@{text c} & @{text "\"} & + @{command "fix"}~@{text x}~@{command "assume"}~@{text "c: \"} \\ + @{command "sorry"} & @{text "\"} & + @{command "by"}~@{text cheating} \\ + \end{tabular} *}