Isabelle_DOF/examples/math_exam/MathExam.thy

65 lines
1.6 KiB
Plaintext
Raw Normal View History

2018-04-17 14:43:08 +00:00
theory MathExam
imports "../../ontologies/mathex_onto"
2018-05-29 10:02:13 +00:00
Real
2018-04-17 14:43:08 +00:00
begin
2018-04-17 14:43:08 +00:00
open_monitor*[exam::MathExam]
2018-05-02 07:40:47 +00:00
section*[idir::Author, affiliation="''CentraleSupelec''",
email="''idir.aitsadoune@centralesupelec.fr''"]
2018-04-27 09:33:47 +00:00
{*Idir AIT SADOUNE*}
2018-04-17 14:43:08 +00:00
2018-05-02 07:40:47 +00:00
subsection*[header::Header,examSubject= "algebra", examTitle="''Exam number 1''",
date="''02-05-2018''", timeAllowed="90::int"]
2018-04-30 11:13:53 +00:00
{*
\begin{itemize}
\item Use black ink or black ball-point pen.
\item Draw diagrams in pencil.
\item Answer all questions in the spaces provided.
\end{itemize}
*}
2018-04-18 07:36:21 +00:00
2018-05-29 10:02:13 +00:00
(*
text*[fig1::figure, width = "Some(textwidth 80)",
"file"="@{file ''../../../figures/Dogfood-Intro.png''}"]
{* Ouroboros I : This paper from inside ... *}
*)
subsubsection*[exo1 :: Exercise, Exercise.content="[q1::Task,q2::Task]"]
2018-04-30 11:13:53 +00:00
{*
Here are the first four lines of a number pattern.
\begin{itemize}
2018-04-30 11:13:53 +00:00
\item Line 1 : @{term "1*6 + 2*4 = 2*7"}
\item Line 2 : @{term "2*7 + 2*5 = 3*8"}
\item Line 3 : @{term "3*8 + 2*6 = 4*9"}
\item Line 4 : @{term "4*9 + 2*7 = 5*10"}
\end{itemize}
2018-04-17 14:43:08 +00:00
*}
2018-05-29 10:02:13 +00:00
lemma XX : "(x ^ 3) + 2 * (x^2) + 11 * x - 12 = (x-4) * (x+1) * (x - 3)"
proof -
have " (x ^ 3) + 2 * (x^2) + 11 * x - 12 = (x + 1) * ( x ^ 2 - 2 * x - 3)"
sorry
have "... = (x + 1) * (x + 4) * (x - 3)"
sorry
show ?thesis
sorry
qed
text*[q1::Task, level="oneStar", mark="1::int", type="formal"]
2018-04-30 11:13:53 +00:00
{*
Complete Line 10 : @{term "10*x + 2*y = 11*16"}
*}
2018-05-29 10:02:13 +00:00
text*[q2::Task, level="threeStars", mark="3::int", type="formal"]
2018-04-17 14:43:08 +00:00
{*
2018-04-30 11:13:53 +00:00
Prove that @{term "n*(n+5) + 2*(n+3) "} is always the product of two numbers with a difference of 5.
2018-04-17 14:43:08 +00:00
*}
2018-04-18 07:36:21 +00:00
close_monitor*[exam]
end