doc-src/TutorialI/Documents/Documents.thy
changeset 14353 79f9fbef9106
parent 13439 2f98365f57a8
child 14486 74c053a25513
equal deleted inserted replaced
14352:a8b1a44d8264 14353:79f9fbef9106
   761   than they really were.  For example, this ``fully automatic'' proof
   761   than they really were.  For example, this ``fully automatic'' proof
   762   is actually a fake:
   762   is actually a fake:
   763 *}
   763 *}
   764 
   764 
   765 lemma "x \<noteq> (0::int) \<Longrightarrow> 0 < x * x"
   765 lemma "x \<noteq> (0::int) \<Longrightarrow> 0 < x * x"
   766   by (auto(*<*)simp add: int_less_le(*>*))
   766   by (auto(*<*)simp add: zero_less_mult_iff(*>*))
   767 
   767 
   768 text {*
   768 text {*
   769   \noindent Here the real source of the proof has been as follows:
   769   \noindent Here the real source of the proof has been as follows:
   770 
   770 
   771 \begin{verbatim}
   771 \begin{verbatim}
   772   by (auto(*<*)simp add: int_less_le(*>*))
   772   by (auto(*<*)simp add: zero_less_mult_iff(*>*))
   773 \end{verbatim}
   773 \end{verbatim}
   774 %(*
   774 %(*
   775 
   775 
   776   \medskip Suppressing portions of printed text demands care.  You
   776   \medskip Suppressing portions of printed text demands care.  You
   777   should not misrepresent the underlying theory development.  It is
   777   should not misrepresent the underlying theory development.  It is