This commit is contained in:
Burkhart Wolff 2018-05-29 14:13:49 +02:00
parent 1fd4f76fb3
commit 37123100df
1 changed files with 7 additions and 3 deletions

View File

@ -36,7 +36,10 @@ Here are the first four lines of a number pattern.
\end{itemize}
*}
lemma check : fixes x::real
(* a bit brutal, as long as lemma* does not yet work *)
(*<*)
lemma check_polynome :
fixes x::real
shows "(x^3) - 6 * x^2 + 5 * x + 12 = (x-4) * (x+1) * (x - 3)"
proof -
@ -51,6 +54,7 @@ proof -
show ?thesis
by(simp only: * ** ***)
qed
(*>*)
text*[a1::Answer_Formal_Step]{* First Step: Fill in term and justification *}
text*[a2::Answer_Formal_Step]{* Next Step: Fill in term and justification *}