author | Andreas Lochbihler |
Wed, 08 Oct 2014 09:09:12 +0200 | |
changeset 58626 | 6c473ed0ac70 |
parent 58520 | a4d1f8041af0 |
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