src/HOL/Nominal/Examples/Nominal_Examples.thy
author wenzelm
Tue, 11 Nov 2014 18:16:25 +0100
changeset 58978 e42da880c61e
parent 58889 5b7a9633cfa8
permissions -rw-r--r--
more position information, e.g. relevant for errors in generated ML source;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
32635
37e32f8aa696 added session theory for Nominal_Examples
haftmann
parents: 28654
diff changeset
     1
(*  Author:  Christian Urban TU Muenchen *)
19495
3d04b87ad8ba New ROOT file for nominal datatype examples.
berghofe
parents:
diff changeset
     2
58889
5b7a9633cfa8 modernized header uniformly as section;
wenzelm
parents: 58329
diff changeset
     3
section {* Various examples involving nominal datatypes. *}
19495
3d04b87ad8ba New ROOT file for nominal datatype examples.
berghofe
parents:
diff changeset
     4
32635
37e32f8aa696 added session theory for Nominal_Examples
haftmann
parents: 28654
diff changeset
     5
theory Nominal_Examples
58329
a31404ec7414 run larger nominal examples only 'ISABELLE_FULL_TEST'
blanchet
parents: 37358
diff changeset
     6
imports Nominal_Examples_Base Class3
32635
37e32f8aa696 added session theory for Nominal_Examples
haftmann
parents: 28654
diff changeset
     7
begin
24895
7cbb842aa99e added two new example files
urbanc
parents: 24153
diff changeset
     8
32635
37e32f8aa696 added session theory for Nominal_Examples
haftmann
parents: 28654
diff changeset
     9
end