src/HOL/ex/svc_test.thy
changeset 7180 35676093459d
child 12873 d7f8dfaad46d
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/ex/svc_test.thy	Fri Aug 06 11:05:20 1999 +0200
@@ -0,0 +1,9 @@
+svc_test = Main +
+
+syntax
+    "<->"         :: [bool, bool] => bool                  (infixr 25)
+
+translations
+  "x <-> y" => "x = y"
+
+end