16 |
16 |
17 session "HOL-Proofs" (slow) = Pure + |
17 session "HOL-Proofs" (slow) = Pure + |
18 description {* |
18 description {* |
19 HOL-Main with explicit proof terms. |
19 HOL-Main with explicit proof terms. |
20 *} |
20 *} |
21 options [document = false, quick_and_dirty = false] |
21 options [condition = ML_SYSTEM_POLYML, document = false, quick_and_dirty = false] |
22 theories Proofs (*sequential change of global flag!*) |
22 theories Proofs (*sequential change of global flag!*) |
23 theories "~~/src/HOL/Library/Old_Datatype" |
23 theories "~~/src/HOL/Library/Old_Datatype" |
24 files |
24 files |
25 "Tools/Quickcheck/Narrowing_Engine.hs" |
25 "Tools/Quickcheck/Narrowing_Engine.hs" |
26 "Tools/Quickcheck/PNF_Narrowing_Engine.hs" |
26 "Tools/Quickcheck/PNF_Narrowing_Engine.hs" |
250 Generate |
250 Generate |
251 Generate_Binary_Nat |
251 Generate_Binary_Nat |
252 Generate_Target_Nat |
252 Generate_Target_Nat |
253 Generate_Efficient_Datastructures |
253 Generate_Efficient_Datastructures |
254 Generate_Pretty_Char |
254 Generate_Pretty_Char |
255 theories [condition = ISABELLE_GHC] |
255 theories [condition = "ML_SYSTEM_POLYML,ISABELLE_GHC"] |
256 Code_Test_GHC |
256 Code_Test_GHC |
257 theories [condition = ISABELLE_MLTON] |
257 theories [condition = "ML_SYSTEM_POLYML,ISABELLE_MLTON"] |
258 Code_Test_MLton |
258 Code_Test_MLton |
259 theories [condition = ISABELLE_OCAMLC] |
259 theories [condition = "ML_SYSTEM_POLYML,ISABELLE_OCAMLC"] |
260 Code_Test_OCaml |
260 Code_Test_OCaml |
261 theories [condition = ISABELLE_POLYML] |
261 theories [condition = "ML_SYSTEM_POLYML,ISABELLE_POLYML"] |
262 Code_Test_PolyML |
262 Code_Test_PolyML |
263 theories [condition = ISABELLE_SCALA] |
263 theories [condition = "ML_SYSTEM_POLYML,ISABELLE_SCALA"] |
264 Code_Test_Scala |
264 Code_Test_Scala |
265 theories [condition = ISABELLE_SMLNJ] |
265 theories [condition = "ML_SYSTEM_POLYML,ISABELLE_SMLNJ"] |
266 Code_Test_SMLNJ |
266 Code_Test_SMLNJ |
267 |
267 |
268 session "HOL-Metis_Examples" in Metis_Examples = HOL + |
268 session "HOL-Metis_Examples" in Metis_Examples = HOL + |
269 description {* |
269 description {* |
270 Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
270 Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
396 *} |
396 *} |
397 options [condition = ML_SYSTEM_POLYML, document = false] |
397 options [condition = ML_SYSTEM_POLYML, document = false] |
398 theories Decision_Procs |
398 theories Decision_Procs |
399 |
399 |
400 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" + |
400 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" + |
401 options [document = false, parallel_proofs = 0] |
401 options [condition = ML_SYSTEM_POLYML, document = false, parallel_proofs = 0] |
402 theories |
402 theories |
403 Hilbert_Classical |
403 Hilbert_Classical |
404 XML_Data |
404 XML_Data |
405 |
405 |
406 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" + |
406 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" + |
430 proves confluence of beta, eta and beta+eta. |
430 proves confluence of beta, eta and beta+eta. |
431 |
431 |
432 The paper "More Church-Rosser Proofs (in Isabelle/HOL)" describes the whole |
432 The paper "More Church-Rosser Proofs (in Isabelle/HOL)" describes the whole |
433 theory (see http://www.in.tum.de/~nipkow/pubs/jar2001.html). |
433 theory (see http://www.in.tum.de/~nipkow/pubs/jar2001.html). |
434 *} |
434 *} |
435 options [print_mode = "no_brackets", parallel_proofs = 0, quick_and_dirty = false] |
435 options [condition = ML_SYSTEM_POLYML, print_mode = "no_brackets", |
|
436 parallel_proofs = 0, quick_and_dirty = false] |
436 theories [document = false] |
437 theories [document = false] |
437 "~~/src/HOL/Library/Code_Target_Int" |
438 "~~/src/HOL/Library/Code_Target_Int" |
438 theories |
439 theories |
439 Eta |
440 Eta |
440 StrongNorm |
441 StrongNorm |
843 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" + |
844 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" + |
844 options [condition = ML_SYSTEM_POLYML, document = false, timeout = 60] |
845 options [condition = ML_SYSTEM_POLYML, document = false, timeout = 60] |
845 theories Ex |
846 theories Ex |
846 |
847 |
847 session "HOL-Word-SMT_Examples" in SMT_Examples = "HOL-Word" + |
848 session "HOL-Word-SMT_Examples" in SMT_Examples = "HOL-Word" + |
848 options [document = false, quick_and_dirty] |
849 options [condition = ML_SYSTEM_POLYML, document = false, quick_and_dirty] |
849 theories |
850 theories |
850 Boogie |
851 Boogie |
851 SMT_Examples |
852 SMT_Examples |
852 SMT_Word_Examples |
853 SMT_Word_Examples |
853 theories [condition = ISABELLE_FULL_TEST] |
854 theories [condition = ISABELLE_FULL_TEST] |
990 Int_Pow |
991 Int_Pow |
991 Lifting_Code_Dt_Test |
992 Lifting_Code_Dt_Test |
992 |
993 |
993 session "HOL-Predicate_Compile_Examples" in Predicate_Compile_Examples = HOL + |
994 session "HOL-Predicate_Compile_Examples" in Predicate_Compile_Examples = HOL + |
994 options [document = false] |
995 options [document = false] |
995 theories |
996 theories [condition = ML_SYSTEM_POLYML] |
996 Examples |
997 Examples |
997 Predicate_Compile_Tests |
998 Predicate_Compile_Tests |
998 Predicate_Compile_Quickcheck_Examples |
999 Predicate_Compile_Quickcheck_Examples |
999 Specialisation_Examples |
1000 Specialisation_Examples |
1000 IMP_1 |
1001 IMP_1 |
1001 IMP_2 |
1002 IMP_2 |
1002 (* FIXME since 21-Jul-2011 |
1003 (* FIXME since 21-Jul-2011 |
1003 Hotel_Example_Small_Generator *) |
1004 Hotel_Example_Small_Generator *) |
1004 IMP_3 |
1005 IMP_3 |
1005 IMP_4 |
1006 IMP_4 |
1006 theories [condition = "ISABELLE_SWIPL"] |
1007 theories [condition = ISABELLE_SWIPL] |
1007 Code_Prolog_Examples |
1008 Code_Prolog_Examples |
1008 Context_Free_Grammar_Example |
1009 Context_Free_Grammar_Example |
1009 Hotel_Example_Prolog |
1010 Hotel_Example_Prolog |
1010 Lambda_Example |
1011 Lambda_Example |
1011 List_Examples |
1012 List_Examples |
1012 theories [condition = "ISABELLE_SWIPL", quick_and_dirty] |
1013 theories [condition = ISABELLE_SWIPL, quick_and_dirty] |
1013 Reg_Exp_Example |
1014 Reg_Exp_Example |
1014 |
1015 |
1015 session HOLCF (main) in HOLCF = HOL + |
1016 session HOLCF (main) in HOLCF = HOL + |
1016 description {* |
1017 description {* |
1017 Author: Franz Regensburger |
1018 Author: Franz Regensburger |