src/HOL/ex/svc_test.thy
author kleing
Mon, 21 Jun 2004 10:25:57 +0200
changeset 14981 e73f8140af78
parent 12873 d7f8dfaad46d
child 17388 495c799df31d
permissions -rw-r--r--
Merged in license change from Isabelle2004


svc_test = SVC_Oracle +

syntax
    "<->"         :: [bool, bool] => bool                  (infixr 25)

translations
  "x <-> y" => "x = y"

end