2454
|
1 |
theory Ex1
|
|
2 |
imports "../Nominal2"
|
2045
|
3 |
begin
|
|
4 |
|
2454
|
5 |
(* free names in bar are bound in foo *)
|
2045
|
6 |
|
|
7 |
atom_decl name
|
|
8 |
|
2561
|
9 |
declare [[STEPS = 100]]
|
|
10 |
|
2045
|
11 |
nominal_datatype foo =
|
|
12 |
Foo0 "name"
|
2436
|
13 |
| Foo1 b::"bar" f::"foo" bind (set) "bv b" in f
|
2045
|
14 |
and bar =
|
|
15 |
Bar0 "name"
|
2436
|
16 |
| Bar1 "name" s::"name" b::"bar" bind (set) s in b
|
2045
|
17 |
binder
|
|
18 |
bv
|
|
19 |
where
|
|
20 |
"bv (Bar0 x) = {}"
|
|
21 |
| "bv (Bar1 v x b) = {atom v}"
|
|
22 |
|
2593
25dcb2b1329e
ordered raw_bn_info to agree with the order of the raw_bn_functions; started alpha_bn proof
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
23 |
thm foo_bar.perm_bn_alpha
|
25dcb2b1329e
ordered raw_bn_info to agree with the order of the raw_bn_functions; started alpha_bn proof
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
24 |
thm foo_bar.perm_bn_simps
|
25dcb2b1329e
ordered raw_bn_info to agree with the order of the raw_bn_functions; started alpha_bn proof
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
25 |
thm foo_bar.bn_finite
|
25dcb2b1329e
ordered raw_bn_info to agree with the order of the raw_bn_functions; started alpha_bn proof
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
26 |
|
25dcb2b1329e
ordered raw_bn_info to agree with the order of the raw_bn_functions; started alpha_bn proof
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
27 |
thm foo_bar.eq_iff
|
2475
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
28 |
thm foo_bar.distinct
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
29 |
thm foo_bar.induct
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
30 |
thm foo_bar.inducts
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
31 |
thm foo_bar.exhaust
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
32 |
thm foo_bar.fv_defs
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
33 |
thm foo_bar.bn_defs
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
34 |
thm foo_bar.perm_simps
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
35 |
thm foo_bar.eq_iff
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
36 |
thm foo_bar.fv_bn_eqvt
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
37 |
thm foo_bar.size_eqvt
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
38 |
thm foo_bar.supports
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
39 |
thm foo_bar.fsupp
|
486d4647bb37
supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
40 |
thm foo_bar.supp
|
2454
|
41 |
|
|
42 |
lemma
|
|
43 |
"fv_foo (Foo1 (Bar1 v x (Bar0 x)) (Foo0 v)) = {}"
|
|
44 |
apply(simp only: foo_bar.fv_defs)
|
|
45 |
apply(simp only: foo_bar.bn_defs)
|
|
46 |
apply(simp only: supp_at_base)
|
|
47 |
apply(simp)
|
|
48 |
done
|
2082
0854af516f14
cleaned up a bit the examples; added equivariance to all examples
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
49 |
|
2045
|
50 |
end
|
|
51 |
|
|
52 |
|