ProgTutorial/Tactical.thy
changeset 307 f4fa6540e280
parent 305 2ac9dc1a95b4
child 308 c90f4ec30d43
equal deleted inserted replaced
306:fe732e890d87 307:f4fa6540e280
  1057 
  1057 
  1058 text {*
  1058 text {*
  1059   will solve all trivial subgoals involving @{term True} or @{term "False"}.
  1059   will solve all trivial subgoals involving @{term True} or @{term "False"}.
  1060 
  1060 
  1061   (FIXME: say something about @{ML [index] COND} and COND')
  1061   (FIXME: say something about @{ML [index] COND} and COND')
       
  1062 
       
  1063   (FIXME: PARALLEL-CHOICE PARALLEL-GOALS)
  1062   
  1064   
  1063   \begin{readmore}
  1065   \begin{readmore}
  1064   Most tactic combinators described in this section are defined in @{ML_file "Pure/tactical.ML"}.
  1066   Most tactic combinators described in this section are defined in @{ML_file "Pure/tactical.ML"}.
  1065   Some combinators for the purpose of proof search are implemented in @{ML_file "Pure/search.ML"}.
  1067   Some combinators for the purpose of proof search are implemented in @{ML_file "Pure/search.ML"}.
  1066   \end{readmore}
  1068   \end{readmore}