src/Doc/IsarImplementation/Tactic.thy
changeset 55547 384bfd19ee61
parent 53096 e79afad81386
equal deleted inserted replaced
55546:76979adf0b96 55547:384bfd19ee61
   918 
   918 
   919   \item @{ML has_fewer_prems}~@{text "n thm"} reports whether @{text
   919   \item @{ML has_fewer_prems}~@{text "n thm"} reports whether @{text
   920   "thm"} has fewer than @{text "n"} premises.
   920   "thm"} has fewer than @{text "n"} premises.
   921 
   921 
   922   \item @{ML Thm.eq_thm}~@{text "(thm\<^sub>1, thm\<^sub>2)"} reports whether @{text
   922   \item @{ML Thm.eq_thm}~@{text "(thm\<^sub>1, thm\<^sub>2)"} reports whether @{text
   923   "thm\<^sub>1"} and @{text "thm\<^sub>2"} are equal.  Both theorems must have
   923   "thm\<^sub>1"} and @{text "thm\<^sub>2"} are equal.  Both theorems must have the
   924   compatible background theories.  Both theorems must have the same
   924   same conclusions, the same set of hypotheses, and the same set of sort
   925   conclusions, the same set of hypotheses, and the same set of sort
       
   926   hypotheses.  Names of bound variables are ignored as usual.
   925   hypotheses.  Names of bound variables are ignored as usual.
   927 
   926 
   928   \item @{ML Thm.eq_thm_prop}~@{text "(thm\<^sub>1, thm\<^sub>2)"} reports whether
   927   \item @{ML Thm.eq_thm_prop}~@{text "(thm\<^sub>1, thm\<^sub>2)"} reports whether
   929   the propositions of @{text "thm\<^sub>1"} and @{text "thm\<^sub>2"} are equal.
   928   the propositions of @{text "thm\<^sub>1"} and @{text "thm\<^sub>2"} are equal.
   930   Names of bound variables are ignored.
   929   Names of bound variables are ignored.