changeset 42208 | 02513eb26eb7 |
parent 42187 | b4f4ed5b8586 |
child 42463 | f270e3e18be5 |
42207:2bda5eddadf3 | 42208:02513eb26eb7 |
---|---|
1 theory Examples |
1 theory Examples |
2 imports Main "~~/src/HOL/Library/Predicate_Compile_Alternative_Defs" |
2 imports Main "~~/src/HOL/Library/Predicate_Compile_Alternative_Defs" |
3 begin |
3 begin |
4 |
4 |
5 declare [[values_timeout = 240.0]] |
5 declare [[values_timeout = 480.0]] |
6 |
6 |
7 section {* Formal Languages *} |
7 section {* Formal Languages *} |
8 |
8 |
9 subsection {* General Context Free Grammars *} |
9 subsection {* General Context Free Grammars *} |
10 |
10 |