doc-src/IsarImplementation/Thy/prelim.thy
changeset 18554 bff7a1466fe4
parent 18537 2681f9e34390
child 20205 7b2958d3d575
--- a/doc-src/IsarImplementation/Thy/prelim.thy	Tue Jan 03 11:57:33 2006 +0100
+++ b/doc-src/IsarImplementation/Thy/prelim.thy	Tue Jan 03 13:59:55 2006 +0100
@@ -189,23 +189,20 @@
 like wood or stone.
 
 Isabelle/Isar distinguishes two key notions of context: \emph{theory
-  context}\indexbold{theory context} and \emph{proof context}.\indexbold{proof
-  context} To motivate this fundamental division consider the very idea of
-logical reasoning which is about judgments $\Gamma \Drv{\Theta} \phi$, where
-$\Theta$ is the background theory with declarations of operators and axioms
-stating their properties, and $\Gamma$ a collection of hypotheses emerging
-temporarily during proof.  For example, the rule of implication-introduction
-\[
-\infer{\Gamma \Drv{\Theta} A \Imp B}{\Gamma, A \Drv{\Theta} B}
-\]
-can be read as ``to show $A \Imp B$ we may assume $A$ as hypothesis and need
-to show $B$''.  It is characteristic that $\Theta$ is unchanged and $\Gamma$
-is only modified according to some general patterns of ``assuming'' and
-``discharging'' hypotheses.  This admits the following abbreviated notation,
-where the fixed $\Theta$ and locally changed $\Gamma$ are left implicit:
-\[
-\infer{A \Imp B}{\infer*{B}{[A]}}
-\]
+context} and \emph{proof context}.  To motivate this fundamental
+division consider the very idea of logical reasoning which is about
+judgments $\Gamma \Drv{\Theta} \phi$, where $\Theta$ is the background
+theory with declarations of operators and axioms stating their
+properties, and $\Gamma$ a collection of hypotheses emerging
+temporarily during proof.  For example, the rule of
+implication-introduction \[ \infer{\Gamma \Drv{\Theta} A \Imp
+B}{\Gamma, A \Drv{\Theta} B} \] can be read as ``to show $A \Imp B$ we
+may assume $A$ as hypothesis and need to show $B$''.  It is
+characteristic that $\Theta$ is unchanged and $\Gamma$ is only
+modified according to some general patterns of ``assuming'' and
+``discharging'' hypotheses.  This admits the following abbreviated
+notation, where the fixed $\Theta$ and locally changed $\Gamma$ are
+left implicit: \[ \infer{A \Imp B}{\infer*{B}{[A]}} \]
 
 In some logical traditions (e.g.\ Type Theory) there is a tendency to
 unify all kinds of declarations within a single notion of context.