| author | blanchet |
| Thu, 28 Aug 2014 00:40:37 +0200 | |
| changeset 58055 | 625bdd5c70b2 |
| parent 58039 | 469a375212c1 |
| child 58348 | 2d47c7d10b62 |
| permissions | -rw-r--r-- |
| 58039 | 1 |
(* Title: Code_Test_PolyML.thy |
2 |
Author: Andreas Lochbihler, ETH Zurich |
|
3 |
||
4 |
Test case for test_code on PolyML |
|
5 |
*) |
|
6 |
||
7 |
theory Code_Test_PolyML imports Code_Test begin |
|
8 |
||
9 |
test_code "14 + 7 * -12 = (140 div -2 :: integer)" in PolyML |
|
10 |
||
11 |
eval_term "14 + 7 * -12 :: integer" in PolyML |
|
12 |
||
13 |
end |