src/HOL/Codegenerator_Test/Code_Test_Scala.thy
changeset 65552 f533820e7248
parent 63167 0909deb8059b
child 66453 cc19f7ca2ed6
equal deleted inserted replaced
65551:d164c4fc0d2c 65552:f533820e7248
     2     Author:     Andreas Lochbihler, ETH Zurich
     2     Author:     Andreas Lochbihler, ETH Zurich
     3 
     3 
     4 Test case for test_code on Scala
     4 Test case for test_code on Scala
     5 *)
     5 *)
     6 
     6 
     7 theory Code_Test_Scala imports  "../Library/Code_Test" "../GCD" begin 
     7 theory Code_Test_Scala imports  "../Library/Code_Test" begin
     8 
     8 
     9 declare [[scala_case_insensitive]]
     9 declare [[scala_case_insensitive]]
    10 
    10 
    11 test_code "14 + 7 * -12 = (140 div -2 :: integer)" in Scala
    11 test_code "14 + 7 * -12 = (140 div -2 :: integer)" in Scala
    12 
    12