src/HOL/ex/svc_test.thy
author wenzelm
Sat, 08 Apr 2006 22:51:28 +0200
changeset 19371 32fc9743803a
parent 17416 5093a587da16
child 20807 bd3b60f9a343
permissions -rw-r--r--
add_abbrevs(_i): support print mode; pretty_term': expand abbreviations only for well-typed terms; added expand_abbrevs; tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
12873
d7f8dfaad46d include SVC_Test;
wenzelm
parents: 7180
diff changeset
     1
17388
495c799df31d tuned headers etc.;
wenzelm
parents: 12873
diff changeset
     2
(* $Id$ *)
495c799df31d tuned headers etc.;
wenzelm
parents: 12873
diff changeset
     3
495c799df31d tuned headers etc.;
wenzelm
parents: 12873
diff changeset
     4
header {* Demonstrating the interface SVC *}
495c799df31d tuned headers etc.;
wenzelm
parents: 12873
diff changeset
     5
495c799df31d tuned headers etc.;
wenzelm
parents: 12873
diff changeset
     6
theory svc_test
495c799df31d tuned headers etc.;
wenzelm
parents: 12873
diff changeset
     7
imports SVC_Oracle
495c799df31d tuned headers etc.;
wenzelm
parents: 12873
diff changeset
     8
begin
7180
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
     9
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
    10
syntax
17416
5093a587da16 fixed type;
wenzelm
parents: 17388
diff changeset
    11
  "<->" :: "[bool, bool] => bool"    (infixr 25)
7180
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
    12
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
    13
translations
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
    14
  "x <-> y" => "x = y"
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
    15
35676093459d new theory ex/svc_test.thy
paulson
parents:
diff changeset
    16
end