1595
|
1 |
theory TestMorePerm
|
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
2 |
imports "../NewParser"
|
1595
|
3 |
begin
|
|
4 |
|
1793
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
5 |
text {*
|
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
6 |
"Weirdo" example from Peter Sewell's bestiary.
|
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
7 |
|
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
8 |
This example is not covered by our binding
|
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
9 |
specification.
|
1595
|
10 |
|
1793
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
11 |
*}
|
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
12 |
ML {* val _ = cheat_equivp := true *}
|
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
13 |
|
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
14 |
atom_decl name
|
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
15 |
|
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
16 |
nominal_datatype weird =
|
1793
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
17 |
Foo_var "name"
|
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
18 |
| Foo_pair "weird" "weird"
|
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
19 |
| Foo x::"name" y::"name" p1::"weird" p2::"weird" p3::"weird"
|
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
20 |
bind x in p1 p2,
|
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
21 |
bind y in p2 p3
|
1793
33f7201a0239
check whether the "weirdo" example from the binding bestiary works with shallow binders
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
22 |
|
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
23 |
thm alpha_weird_raw.intros[no_vars]
|
1595
|
24 |
|
|
25 |
thm permute_weird_raw.simps[no_vars]
|
|
26 |
thm alpha_weird_raw.intros[no_vars]
|
|
27 |
thm fv_weird_raw.simps[no_vars]
|
|
28 |
|
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
29 |
equivariance alpha_weird_raw
|
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
30 |
|
1595
|
31 |
|
|
32 |
end
|
|
33 |
|
|
34 |
|
|
35 |
|