src/HOL/ex/svc_test.thy
author huffman
Wed, 06 Jul 2005 00:08:57 +0200
changeset 16701 abd0abd66387
parent 12873 d7f8dfaad46d
child 17388 495c799df31d
permissions -rw-r--r--
add keywords cpodef, pcpodef (for HOLCF)
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
12873
d7f8dfaad46d include SVC_Test;
wenzelm
parents: 7180
diff changeset
     1
d7f8dfaad46d include SVC_Test;
wenzelm
parents: 7180
diff changeset
     2
svc_test = SVC_Oracle +
7180
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     3
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     4
syntax
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     5
    "<->"         :: [bool, bool] => bool                  (infixr 25)
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     6
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     7
translations
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     8
  "x <-> y" => "x = y"
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     9
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
    10
end