| author | hoelzl |
| Mon, 24 Nov 2014 12:20:14 +0100 | |
| changeset 59048 | 7dc8ac6f0895 |
| parent 58626 | 6c473ed0ac70 |
| child 59720 | f893472fff31 |
| permissions | -rw-r--r-- |
(* Title: Code_Test_Scala.thy Author: Andreas Lochbihler, ETH Zurich Test case for test_code on Scala *) theory Code_Test_Scala imports "../Library/Code_Test" begin declare [[scala_case_insensitive]] test_code "14 + 7 * -12 = (140 div -2 :: integer)" in Scala value [Scala] "14 + 7 * -12 :: integer" end