src/HOL/Nominal/Examples/Nominal_Examples.thy
author wenzelm
Tue, 20 Apr 2010 11:26:25 +0200
changeset 36212 ebfa4bb0d50f
parent 33189 82a40677c1f8
child 36277 9be4ab2acc13
permissions -rw-r--r--
refer to THIS_JAVA dynamically, and treat ISABELLE_JAVA as static default -- relevant for nested JVM invocation within an existing Isabelle enviroment;

(*  Author:  Christian Urban TU Muenchen *)

header {* Various examples involving nominal datatypes. *}

theory Nominal_Examples
imports
  CR
  CR_Takahashi
  Class
  Compile
  Fsub
  Height
  Lambda_mu
  SN
  Weakening
  Crary
  SOS
  LocalWeakening
  Support
  Contexts
  Standardization
  W
  Pattern
begin

end