ProgTutorial/Recipes/TimeLimit.thy
author Norbert Schirmer <norbert.schirmer@web.de>
Tue, 14 May 2019 11:10:53 +0200
changeset 562 daf404920ab9
parent 557 77ea2de0ca62
child 565 cecd7a941885
permissions -rw-r--r--
Accomodate to Isabelle 2018
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
     1
theory TimeLimit
346
0fea8b7a14a1 tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents: 191
diff changeset
     2
imports "../Appendix"
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
     3
begin
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
     4
94
531e453c9d67 rewrote recipes describing external solvers
boehmes
parents: 72
diff changeset
     5
section {* Restricting the Runtime of a Function\label{rec:timeout} *} 
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
     6
text {*
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
     7
  {\bf Problem:}
63
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
     8
  Your tool should run only a specified amount of time.\smallskip
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
     9
562
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    10
  {\bf Solution:} In Isabelle 2016-1 and later, this can be achieved 
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    11
  using the function @{ML apply in Timeout}.\smallskip
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
    12
168
009ca4807baa polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents: 155
diff changeset
    13
  Assume you defined the Ackermann function on the ML-level.
009ca4807baa polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents: 155
diff changeset
    14
*}
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
    15
517
d8c376662bb4 removed special ML-setup and replaced it by explicit markups (i.e., %grayML)
Christian Urban <urbanc@in.tum.de>
parents: 346
diff changeset
    16
ML %grayML{*fun ackermann (0, n) = n + 1
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
    17
  | ackermann (m, 0) = ackermann (m - 1, 1)
69
19106a9975c1 highligted the background of ML-code
Christian Urban <urbanc@in.tum.de>
parents: 68
diff changeset
    18
  | ackermann (m, n) = ackermann (m - 1, ackermann (m, n - 1)) *}
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
    19
63
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    20
text {*
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    21
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    22
  Now the call 
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    23
557
77ea2de0ca62 updated for Isabelle 2014
Christian Urban <christian dot urban at kcl dot ac dot uk>
parents: 517
diff changeset
    24
  @{ML_response_fake_both [display,gray] "ackermann (4, 12)" "\<dots>"}
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
    25
68
e7519207c2b7 added more to the "new command section" and tuning
Christian Urban <urbanc@in.tum.de>
parents: 67
diff changeset
    26
  takes a bit of time before it finishes. To avoid this, the call can be encapsulated 
168
009ca4807baa polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents: 155
diff changeset
    27
  in a time limit of five seconds. For this you have to write
63
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    28
186
371e4375c994 made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
parents: 175
diff changeset
    29
@{ML_response_fake_both [display,gray]
562
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    30
"Timeout.apply (Time.fromSeconds 5) ackermann (4, 12) 
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    31
  handle TIMEOUT => ~1"
63
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    32
"~1"}
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
    33
102
5e309df58557 general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
parents: 94
diff changeset
    34
  where @{text TimeOut} is the exception raised when the time limit
63
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    35
  is reached.
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    36
562
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    37
  Note that @{ML  "apply" in Timeout} is only meaningful when you use PolyML 5.2.1
186
371e4375c994 made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
parents: 175
diff changeset
    38
  or later, because this version of PolyML has the infrastructure for multithreaded 
562
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    39
  programming on which @{ML "apply" in Timeout} relies.
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
    40
63
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    41
\begin{readmore}
562
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    42
   The function @{ML "apply" in Timeout} is defined in the structure
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    43
  @{ML_struct Timeout} which can be found in the file 
daf404920ab9 Accomodate to Isabelle 2018
Norbert Schirmer <norbert.schirmer@web.de>
parents: 557
diff changeset
    44
  @{ML_file "Pure/concurrent/timeout.ML"}.
63
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    45
\end{readmore}
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    46
Christian Urban <urbanc@in.tum.de>
parents: 61
diff changeset
    47
 
61
64c9540f2f84 Added four recipes.
boehmes
parents:
diff changeset
    48
*}
517
d8c376662bb4 removed special ML-setup and replaced it by explicit markups (i.e., %grayML)
Christian Urban <urbanc@in.tum.de>
parents: 346
diff changeset
    49
end