src/HOL/ex/svc_test.thy
author wenzelm
Wed, 14 Sep 2005 22:08:08 +0200
changeset 17388 495c799df31d
parent 12873 d7f8dfaad46d
child 17416 5093a587da16
permissions -rw-r--r--
tuned headers etc.;


(* $Id$ *)

header {* Demonstrating the interface SVC *}

theory svc_test
imports SVC_Oracle
begin

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

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

end