reactivated Scala check; tuned import order
authorhaftmann
Mon, 26 Jul 2010 11:09:45 +0200
changeset 37967 3e174df3f965
parent 37966 ac9bcae5ada7
child 37968 52fdcb76c0af
reactivated Scala check; tuned import order
src/HOL/Imperative_HOL/ex/Imperative_Reverse.thy
--- a/src/HOL/Imperative_HOL/ex/Imperative_Reverse.thy	Mon Jul 26 11:09:45 2010 +0200
+++ b/src/HOL/Imperative_HOL/ex/Imperative_Reverse.thy	Mon Jul 26 11:09:45 2010 +0200
@@ -5,7 +5,7 @@
 header {* An imperative in-place reversal on arrays *}
 
 theory Imperative_Reverse
-imports Imperative_HOL Subarray
+imports Subarray Imperative_HOL
 begin
 
 fun swap :: "'a\<Colon>heap array \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> unit Heap" where
@@ -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