src/Doc/Implementation/Eq.thy
changeset 61458 987533262fc2
parent 61439 2bf52eec4e8a
child 61493 0debd22f0c0e
--- a/src/Doc/Implementation/Eq.thy	Fri Oct 16 10:11:20 2015 +0200
+++ b/src/Doc/Implementation/Eq.thy	Fri Oct 16 14:53:26 2015 +0200
@@ -98,8 +98,6 @@
   @{index_ML fold_goals_tac: "Proof.context -> thm list -> tactic"} \\
   \end{mldecls}
 
-  \begin{description}
-
   \<^descr> @{ML rewrite_rule}~@{text "ctxt rules thm"} rewrites the whole
   theorem by the given rules.
 
@@ -119,8 +117,6 @@
   "rules"}, re-ordered to fold longer expression first.  This supports
   to idea to fold primitive definitions that appear in expended form
   in the proof state.
-
-  \end{description}
 \<close>
 
 end