src/HOL/ex/svc_test.thy
author nipkow
Mon, 13 Mar 2000 12:51:10 +0100
changeset 8423 3c19160b6432
parent 7180 35676093459d
child 12873 d7f8dfaad46d
permissions -rw-r--r--
exhaust_tac -> cases_tac
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
7180
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     1
svc_test = Main +
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     2
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     3
syntax
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     4
    "<->"         :: [bool, bool] => bool                  (infixr 25)
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     5
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     6
translations
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     7
  "x <-> y" => "x = y"
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     8
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     9
end