author | wenzelm |
Fri, 22 Oct 2010 19:03:31 +0100 | |
changeset 39882 | ab0afd03a042 |
parent 39866 | 5ec01d5acd0c |
child 40110 | 93e7935d4cb5 |
permissions | -rw-r--r-- |
29755 | 1 |
theory Base |
39846 | 2 |
imports Main |
21374 | 3 |
uses "../../antiquote_setup.ML" |
18537 | 4 |
begin |
30272 | 5 |
|
39866
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39846
diff
changeset
|
6 |
(* FIXME move to src/Pure/ML/ml_antiquote.ML *) |
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39846
diff
changeset
|
7 |
ML {* |
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39846
diff
changeset
|
8 |
ML_Antiquote.inline "assert" |
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39846
diff
changeset
|
9 |
(Scan.succeed "(fn b => if b then () else raise General.Fail \"Assertion failed\")") |
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39846
diff
changeset
|
10 |
*} |
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39846
diff
changeset
|
11 |
|
18537 | 12 |
end |