src/HOL/ex/svc_test.thy
author paulson
Mon, 22 Oct 2001 11:54:22 +0200
changeset 11868 56db9f3a6b3e
parent 7180 35676093459d
child 12873 d7f8dfaad46d
permissions -rw-r--r--
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite to their abstract counterparts, while other binary numerals work correctly.

svc_test = Main +

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

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

end