src/HOL/HOL.thy
changeset 48073 1b609a7837ef
parent 47657 1ba213363d0c
child 48195 3127f9ce52fb
--- a/src/HOL/HOL.thy	Tue Jun 05 07:05:56 2012 +0200
+++ b/src/HOL/HOL.thy	Tue Jun 05 07:10:51 2012 +0200
@@ -1903,7 +1903,7 @@
   (SML "!(raise/ Fail/ \"undefined\")")
   (OCaml "failwith/ \"undefined\"")
   (Haskell "error/ \"undefined\"")
-  (Scala "!error(\"undefined\")")
+  (Scala "!sys.error(\"undefined\")")
 
 subsubsection {* Evaluation and normalization by evaluation *}