diff -r e4c5c7ffceea -r fee67c099d03 doc-src/IsarImplementation/Thy/Proof.thy --- a/doc-src/IsarImplementation/Thy/Proof.thy Tue May 03 21:40:14 2011 +0200 +++ b/doc-src/IsarImplementation/Thy/Proof.thy Tue May 03 21:44:05 2011 +0200 @@ -253,14 +253,14 @@ \medskip The most basic export rule discharges assumptions directly by means of the @{text "\"} introduction rule: \[ - \infer[(@{text "\\intro"})]{@{text "\ - A \ A \ B"}}{@{text "\ \ B"}} + \infer[(@{text "\\intro"})]{@{text "\ - A \ A \ B"}}{@{text "\ \ B"}} \] The variant for goal refinements marks the newly introduced premises, which causes the canonical Isar goal refinement scheme to enforce unification with local premises within the goal: \[ - \infer[(@{text "#\\intro"})]{@{text "\ - A \ #A \ B"}}{@{text "\ \ B"}} + \infer[(@{text "#\\intro"})]{@{text "\ - A \ #A \ B"}}{@{text "\ \ B"}} \] \medskip Alternative versions of assumptions may perform arbitrary @@ -269,7 +269,7 @@ definition works by fixing @{text "x"} and assuming @{text "x \ t"}, with the following export rule to reverse the effect: \[ - \infer[(@{text "\\expand"})]{@{text "\ - (x \ t) \ B t"}}{@{text "\ \ B x"}} + \infer[(@{text "\\expand"})]{@{text "\ - (x \ t) \ B t"}}{@{text "\ \ B x"}} \] This works, because the assumption @{text "x \ t"} was introduced in a context with @{text "x"} being fresh, so @{text "x"} does not @@ -307,7 +307,7 @@ \item @{ML Assumption.add_assumes}~@{text "As"} is a special case of @{ML Assumption.add_assms} where the export rule performs @{text - "\\intro"} or @{text "#\\intro"}, depending on goal + "\\intro"} or @{text "#\\intro"}, depending on goal mode. \item @{ML Assumption.export}~@{text "is_goal inner outer thm"}