Isabelle_DOF/examples/math_exam/MathExam.thy

46 lines
1.2 KiB
Plaintext
Raw Normal View History

2018-04-17 14:43:08 +00:00
theory MathExam
imports "../../ontologies/mathex_onto"
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-02 07:40:47 +00:00
subsubsection*[exo1 :: Exercise, Exercise.content="[q1::Question,q2::Question]"]
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-04-30 11:13:53 +00:00
text*[q1::Question, level="oneStar", Question.mark="1::int", type="formal"]
{*
Complete Line 10 : @{term "10*x + 2*y = 11*16"}
*}
text*[q2::Question, level="threeStars", Question.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