2045
+ − 1
theory Term8
+ − 2
imports "../NewParser"
+ − 3
begin
+ − 4
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 5
(* example 8 *)
2045
+ − 6
+ − 7
atom_decl name
+ − 8
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 9
(* this should work but gives an error at the moment:
2097
+ − 10
in alpha_bn_rsp proof.
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 11
*)
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 12
2045
+ − 13
nominal_datatype foo =
+ − 14
Foo0 "name"
+ − 15
| Foo1 b::"bar" f::"foo" bind_set "bv b" in f
+ − 16
and bar =
+ − 17
Bar0 "name"
2097
+ − 18
| Bar1 "name" s::"name" b::"bar" bind_set s in b
2045
+ − 19
binder
+ − 20
bv
+ − 21
where
+ − 22
"bv (Bar0 x) = {}"
+ − 23
| "bv (Bar1 v x b) = {atom v}"
+ − 24
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 25
2045
+ − 26
end
+ − 27
+ − 28