src/HOL/Nominal/Examples/Lambda_mu.thy
author wenzelm
Sun, 16 Jan 2011 15:53:03 +0100
changeset 41589 bbd861837ebc
parent 25867 c24395ea4e71
child 63167 0909deb8059b
permissions -rw-r--r--
tuned headers;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
19501
9afa7183dfc2 Capitalized theory names.
berghofe
parents: 18659
diff changeset
     1
theory Lambda_mu 
25867
c24395ea4e71 tuned proofs
urbanc
parents: 22829
diff changeset
     2
  imports "../Nominal" 
18106
836135c8acb2 Initial commit.
urbanc
parents:
diff changeset
     3
begin
836135c8acb2 Initial commit.
urbanc
parents:
diff changeset
     4
18269
3f36e2165e51 some small tuning
urbanc
parents: 18106
diff changeset
     5
section {* Lambda-Mu according to a paper by Gavin Bierman *}
18106
836135c8acb2 Initial commit.
urbanc
parents:
diff changeset
     6
836135c8acb2 Initial commit.
urbanc
parents:
diff changeset
     7
atom_decl var mvar
836135c8acb2 Initial commit.
urbanc
parents:
diff changeset
     8
22829
f1db55c7534d tuned some proofs and changed variable names in some definitions of Nominal.thy
urbanc
parents: 19501
diff changeset
     9
nominal_datatype trm = 
f1db55c7534d tuned some proofs and changed variable names in some definitions of Nominal.thy
urbanc
parents: 19501
diff changeset
    10
    Var   "var" 
f1db55c7534d tuned some proofs and changed variable names in some definitions of Nominal.thy
urbanc
parents: 19501
diff changeset
    11
  | Lam  "\<guillemotleft>var\<guillemotright>trm"   ("Lam [_]._" [100,100] 100)
f1db55c7534d tuned some proofs and changed variable names in some definitions of Nominal.thy
urbanc
parents: 19501
diff changeset
    12
  | App  "trm" "trm" 
25867
c24395ea4e71 tuned proofs
urbanc
parents: 22829
diff changeset
    13
  | Pss  "mvar" "trm"                                   (* passivate *)
c24395ea4e71 tuned proofs
urbanc
parents: 22829
diff changeset
    14
  | Act  "\<guillemotleft>mvar\<guillemotright>trm"  ("Act [_]._" [100,100] 100)       (* activate  *)
c24395ea4e71 tuned proofs
urbanc
parents: 22829
diff changeset
    15
18106
836135c8acb2 Initial commit.
urbanc
parents:
diff changeset
    16
19501
9afa7183dfc2 Capitalized theory names.
berghofe
parents: 18659
diff changeset
    17
end