src/HOL/ex/mesontest2.thy
author wenzelm
Sun, 01 Oct 2006 18:29:32 +0200
changeset 20813 379ce56e5dc2
parent 19668 6afaf300cb78
child 23774 07968f8cc662
permissions -rw-r--r--
proper use of svc_oracle.ML;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
15285
ce83b7e74a91 Renamed some variables to eliminate conflicts with constants.
paulson
parents: 11586
diff changeset
     1
(*ID:         $Id$*)
11586
wenzelm
parents: 10440
diff changeset
     2
header {* Meson test cases *}
10440
2074e62da354 proper theory context for mesontest2;
wenzelm
parents:
diff changeset
     3
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 15285
diff changeset
     4
theory mesontest2 imports Main begin
10440
2074e62da354 proper theory context for mesontest2;
wenzelm
parents:
diff changeset
     5
19668
6afaf300cb78 hide const subst;
wenzelm
parents: 16417
diff changeset
     6
hide const subset
6afaf300cb78 hide const subst;
wenzelm
parents: 16417
diff changeset
     7
10440
2074e62da354 proper theory context for mesontest2;
wenzelm
parents:
diff changeset
     8
end