Nominal/Ex/TestMorePerm.thy
author Cezary Kaliszyk <kaliszyk@in.tum.de>
Mon, 19 Apr 2010 09:59:32 +0200
changeset 1875 0c3fa0cc2d82
parent 1793 33f7201a0239
child 2082 0854af516f14
permissions -rw-r--r--
Locations of files in Parser

theory TestMorePerm
imports "../Parser"
begin

text {* 
  "Weirdo" example from Peter Sewell's bestiary. 

  In case of deep binders, it is not coverd by our 
  approach of defining alpha-equivalence with a 
  single permutation.

  Check whether it works with shallow binders as
  defined below.

*}
ML {* val _ = cheat_equivp := true *}

atom_decl name

nominal_datatype foo =
  Foo_var "name"
| Foo_pair "foo" "foo" 
| Foo x::"name" y::"name" p1::"foo" p2::"foo" p3::"foo"
    bind x in p1, bind x in p2, 
    bind y in p2, bind y in p3

thm alpha_foo_raw.intros[no_vars]

thm permute_weird_raw.simps[no_vars]
thm alpha_weird_raw.intros[no_vars]
thm fv_weird_raw.simps[no_vars]


end