src/HOL/ex/svc_test.thy
author wenzelm
Sat, 07 Jan 2006 12:26:33 +0100
changeset 18608 9cdcc2a5c8b3
parent 17416 5093a587da16
child 20807 bd3b60f9a343
permissions -rw-r--r--
support nested cases; added apply_case; replaced make/simple by make_common/nested/simple;


(* $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