ProgTutorial/FirstSteps.thy
changeset 225 7859fc59249a
parent 215 8d1a344a621e
child 228 fe45fbb111c5
equal deleted inserted replaced
224:647cab4a72c2 225:7859fc59249a
   558 text {* 
   558 text {* 
   559   Now querying the definition you obtain:
   559   Now querying the definition you obtain:
   560 
   560 
   561   \begin{isabelle}
   561   \begin{isabelle}
   562   \isacommand{thm}~@{text "TrueConj_def"}\\
   562   \isacommand{thm}~@{text "TrueConj_def"}\\
   563   @{text "> "}@{thm TrueConj_def}
   563   @{text "> "}~@{thm TrueConj_def}
   564   \end{isabelle}
   564   \end{isabelle}
   565 
   565 
   566   (FIXME give a better example why bindings are important; maybe
   566   (FIXME give a better example why bindings are important; maybe
   567   give a pointer to \isacommand{local\_setup})
   567   give a pointer to \isacommand{local\_setup})
   568 
   568