Nominal/Ex/Test.thy
author Christian Urban <urbanc@in.tum.de>
Wed, 11 Aug 2010 16:21:24 +0800
changeset 2393 d9a0cf26a88c
parent 2288 3b83960f9544
permissions -rw-r--r--
added a function that transforms the helper-rsp lemmas into real rsp lemmas

theory Test
imports "../NewParser"
begin

declare [[STEPS = 4]]

atom_decl name

(*
nominal_datatype trm =
  Vr "name"
| Ap "trm" "trm"

thm fv_trm_raw.simps[no_vars]
*)

(* This file contains only the examples that are not supposed to work yet. *)


declare [[STEPS = 2]]


(* example 4 from Terms.thy *)
(* fv_eqvt does not work, we need to repaire defined permute functions
   defined fv and defined alpha... *)
(* lists-datastructure does not work yet *)

nominal_datatype trm =
  Vr "name"
| Ap "trm" "trm list"
| Lm x::"name" t::"trm"  bind x in t

(*
thm alpha_trm4_raw_alpha_trm4_raw_list.intros[no_vars]
thm fv_trm4_raw_fv_trm4_raw_list.simps[no_vars]
*)

end