src/HOL/ex/svc_test.thy
changeset 17416 5093a587da16
parent 17388 495c799df31d
child 20807 bd3b60f9a343
--- a/src/HOL/ex/svc_test.thy	Thu Sep 15 17:17:03 2005 +0200
+++ b/src/HOL/ex/svc_test.thy	Thu Sep 15 17:17:04 2005 +0200
@@ -8,7 +8,7 @@
 begin
 
 syntax
-    "<->"         :: [bool, bool] => bool                  (infixr 25)
+  "<->" :: "[bool, bool] => bool"    (infixr 25)
 
 translations
   "x <-> y" => "x = y"