src/Doc/Implementation/Tactic.thy
changeset 59902 6afbe5a99139
parent 59780 23b67731f4f0
child 61416 b9a3324e4e62
equal deleted inserted replaced
59901:840d03805755 59902:6afbe5a99139
   707   evaluation in Standard ML.  The following attempt would make @{ML
   707   evaluation in Standard ML.  The following attempt would make @{ML
   708   REPEAT}~@{text "tac"} loop:
   708   REPEAT}~@{text "tac"} loop:
   709   \end{warn}
   709   \end{warn}
   710 \<close>
   710 \<close>
   711 
   711 
   712 ML \<open>
   712 ML_val \<open>
   713   (*BAD -- does not terminate!*)
   713   (*BAD -- does not terminate!*)
   714   fun REPEAT tac = (tac THEN REPEAT tac) ORELSE all_tac;
   714   fun REPEAT tac = (tac THEN REPEAT tac) ORELSE all_tac;
   715 \<close>
   715 \<close>
   716 
   716 
   717 
   717