src/HOL/Nominal/Examples/Lambda_mu.thy
author urbanc
Wed, 11 Jan 2006 18:38:32 +0100
changeset 18659 2ff0ae57431d
parent 18269 3f36e2165e51
child 19501 9afa7183dfc2
permissions -rw-r--r--
changes to make use of the new induction principle proved by Stefan horay (hooraayyy)

(* $Id$ *)

theory lambda_mu 
imports "../nominal" 
begin

section {* Lambda-Mu according to a paper by Gavin Bierman *}

atom_decl var mvar

nominal_datatype trm = Var   "var" 
                     | Lam  "\<guillemotleft>var\<guillemotright>trm"   ("Lam [_]._" [100,100] 100)
                     | App  "trm" "trm" 
                     | Pss  "mvar" "trm"
                     | Act  "\<guillemotleft>mvar\<guillemotright>trm"  ("Act [_]._" [100,100] 100)