diff -r 2995639c6a09 -r 90695f46440b doc-src/TutorialI/Misc/case_exprs.thy --- a/doc-src/TutorialI/Misc/case_exprs.thy Fri Jan 12 16:28:14 2001 +0100 +++ b/doc-src/TutorialI/Misc/case_exprs.thy Fri Jan 12 16:32:01 2001 +0100 @@ -2,7 +2,7 @@ theory case_exprs = Main: (*>*) -subsection{*Case expressions*} +subsection{*Case Expressions*} text{*\label{sec:case-expressions} HOL also features \isaindexbold{case}-expressions for analyzing @@ -40,7 +40,7 @@ indicate their scope *} -subsection{*Structural induction and case distinction*} +subsection{*Structural Induction and Case Distinction*} text{*\label{sec:struct-ind-case} \indexbold{structural induction}