1159
3c6bee89d826
Ported Stefan's permutation code, still needs some localizing.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff
changeset
|
1 |
theory Perm
|
2288
3b83960f9544
new fv/fv_bn function (supp breaks now); exported raw perms and raw funs into separate ML-files
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
2 |
imports
|
3b83960f9544
new fv/fv_bn function (supp breaks now); exported raw perms and raw funs into separate ML-files
Christian Urban <urbanc@in.tum.de>
diff
changeset
|
3 |
"../Nominal-General/Nominal2_Base"
|
2296
|
4 |
"../Nominal-General/Nominal2_Atoms"
|
2302
|
5 |
"../Nominal-General/Nominal2_Eqvt"
|
|
6 |
"Nominal2_FSet"
|
|
7 |
"Abs"
|
2305
|
8 |
uses ("nominal_dt_rawperm.ML")
|
2296
|
9 |
("nominal_dt_rawfuns.ML")
|
2305
|
10 |
("nominal_dt_alpha.ML")
|
2337
|
11 |
("nominal_dt_quot.ML")
|
1159
3c6bee89d826
Ported Stefan's permutation code, still needs some localizing.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff
changeset
|
12 |
begin
|
3c6bee89d826
Ported Stefan's permutation code, still needs some localizing.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
diff
changeset
|
13 |
|
2296
|
14 |
use "nominal_dt_rawperm.ML"
|
2297
|
15 |
ML {* open Nominal_Dt_RawPerm *}
|
2296
|
16 |
|
2297
|
17 |
use "nominal_dt_rawfuns.ML"
|
|
18 |
ML {* open Nominal_Dt_RawFuns *}
|
2296
|
19 |
|
2297
|
20 |
use "nominal_dt_alpha.ML"
|
|
21 |
ML {* open Nominal_Dt_Alpha *}
|
2296
|
22 |
|
2337
|
23 |
use "nominal_dt_quot.ML"
|
|
24 |
ML {* open Nominal_Dt_Quot *}
|
|
25 |
|
|
26 |
|
1903
|
27 |
end
|