doc-src/IsarImplementation/Thy/Isar.thy
author wenzelm
Mon, 16 Feb 2009 20:47:44 +0100
changeset 29755 d66b34e46bdf
parent 20520 doc-src/IsarImplementation/Thy/isar.thy@05fd007bdeb9
child 29759 bcb79ddf57da
permissions -rw-r--r--
observe usual theory naming conventions;

theory Isar
imports Base
begin

chapter {* Isar proof texts *}

section {* Proof context *}

text FIXME


section {* Proof state \label{sec:isar-proof-state} *}

text {*
  FIXME

\glossary{Proof state}{The whole configuration of a structured proof,
consisting of a \seeglossary{proof context} and an optional
\seeglossary{structured goal}.  Internally, an Isar proof state is
organized as a stack to accomodate block structure of proof texts.
For historical reasons, a low-level \seeglossary{tactical goal} is
occasionally called ``proof state'' as well.}

\glossary{Structured goal}{FIXME}

\glossary{Goal}{See \seeglossary{tactical goal} or \seeglossary{structured goal}. \norefpage}


*}

section {* Proof methods *}

text FIXME

section {* Attributes *}

text "FIXME ?!"


end