temporarily deactivating check for Scala
authorhaftmann
Sat, 24 Jul 2010 18:08:43 +0200
changeset 37959 6fe5fa827f18
parent 37958 9728342bcd56
child 37963 61887e5b3d1d
child 37964 0a1ae22df1f1
temporarily deactivating check for Scala
src/HOL/Imperative_HOL/Imperative_HOL_ex.thy
src/HOL/Imperative_HOL/ex/Imperative_Quicksort.thy
src/HOL/Imperative_HOL/ex/Imperative_Reverse.thy
src/HOL/Imperative_HOL/ex/Linked_Lists.thy
--- a/src/HOL/Imperative_HOL/Imperative_HOL_ex.thy	Sat Jul 24 18:08:41 2010 +0200
+++ b/src/HOL/Imperative_HOL/Imperative_HOL_ex.thy	Sat Jul 24 18:08:43 2010 +0200
@@ -14,6 +14,6 @@
   Array.upd, Array.map_entry, Array.swap, Array.freeze,
   ref, Ref.lookup, Ref.update, Ref.change)"
 
-export_code everything checking SML SML_imp OCaml? OCaml_imp? Haskell? Scala?
+export_code everything checking SML SML_imp OCaml? OCaml_imp? Haskell? (*Scala?*)
 
 end
--- a/src/HOL/Imperative_HOL/ex/Imperative_Quicksort.thy	Sat Jul 24 18:08:41 2010 +0200
+++ b/src/HOL/Imperative_HOL/ex/Imperative_Quicksort.thy	Sat Jul 24 18:08:43 2010 +0200
@@ -655,6 +655,6 @@
 
 ML {* @{code qsort} (Array.fromList [42, 2, 3, 5, 0, 1705, 8, 3, 15]) () *}
 
-export_code qsort checking SML SML_imp OCaml? OCaml_imp? Haskell? Scala?
+export_code qsort checking SML SML_imp OCaml? OCaml_imp? Haskell? (*Scala?*)
 
 end
--- a/src/HOL/Imperative_HOL/ex/Imperative_Reverse.thy	Sat Jul 24 18:08:41 2010 +0200
+++ b/src/HOL/Imperative_HOL/ex/Imperative_Reverse.thy	Sat Jul 24 18:08:43 2010 +0200
@@ -110,6 +110,6 @@
       subarray_def sublist'_all rev.simps[where j=0] elim!: crel_elims)
   (drule sym[of "List.length (Array.get h a)"], simp)
 
-export_code rev checking SML SML_imp OCaml? OCaml_imp? Haskell? Scala?
+export_code rev checking SML SML_imp OCaml? OCaml_imp? Haskell? (*Scala?*)
 
 end
--- a/src/HOL/Imperative_HOL/ex/Linked_Lists.thy	Sat Jul 24 18:08:41 2010 +0200
+++ b/src/HOL/Imperative_HOL/ex/Linked_Lists.thy	Sat Jul 24 18:08:43 2010 +0200
@@ -1014,6 +1014,6 @@
 ML {* @{code test_2} () *}
 ML {* @{code test_3} () *}
 
-export_code test_1 test_2 test_3 checking SML SML_imp OCaml? OCaml_imp? Haskell? Scala?
+export_code test_1 test_2 test_3 checking SML SML_imp OCaml? OCaml_imp? Haskell? (*Scala?*)
 
 end