author | Christian Urban <urbanc@in.tum.de> |
Thu, 08 Apr 2010 11:40:13 +0200 | |
changeset 1792 | c29a139410d2 |
parent 1773 | c0eac04ae3b4 |
child 1793 | 33f7201a0239 |
permissions | -rw-r--r-- |
theory TestMorePerm imports "../Parser" begin text {* weirdo example from Peter Sewell's bestiary *} nominal_datatype weird = WBind x::"name" y::"name" p1::"weird" p2::"weird" p3::"weird" bind x in p1, bind x in p2, bind y in p2, bind y in p3 | WV "name" | WP "weird" "weird" thm permute_weird_raw.simps[no_vars] thm alpha_weird_raw.intros[no_vars] thm fv_weird_raw.simps[no_vars] end