author | wenzelm |
Wed, 12 Mar 2025 11:39:00 +0100 | |
changeset 82265 | 4b875a4c83b0 |
parent 81136 | 2b949a3bfaac |
permissions | -rw-r--r-- |
28213 | 1 |
theory Setup |
39066 | 2 |
imports |
3 |
Complex_Main |
|
66453
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents:
61670
diff
changeset
|
4 |
"HOL-Library.Dlist" |
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents:
61670
diff
changeset
|
5 |
"HOL-Library.RBT" |
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents:
61670
diff
changeset
|
6 |
"HOL-Library.Mapping" |
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents:
61670
diff
changeset
|
7 |
"HOL-Library.IArray" |
28213 | 8 |
begin |
9 |
||
69605 | 10 |
ML_file \<open>../antiquote_setup.ML\<close> |
11 |
ML_file \<open>../more_antiquote.ML\<close> |
|
48891 | 12 |
|
81136 | 13 |
unbundle constrain_space_syntax |
38503 | 14 |
|
59324 | 15 |
declare [[default_code_width = 74]] |
34071 | 16 |
|
42669
04dfffda5671
more conventional naming scheme: names_long, names_short, names_unique;
wenzelm
parents:
42358
diff
changeset
|
17 |
declare [[names_unique = false]] |
28213 | 18 |
|
19 |
end |