src/HOL/ROOT
changeset 51143 0a2371e7ced3
parent 51115 7dbd6832a689
child 51160 599ff65b85e2
equal deleted inserted replaced
51142:ac9e909fe55d 51143:0a2371e7ced3
    26     Finite_Lattice
    26     Finite_Lattice
    27     Code_Char_chr
    27     Code_Char_chr
    28     Code_Char_ord
    28     Code_Char_ord
    29     Product_Lexorder
    29     Product_Lexorder
    30     Product_Order
    30     Product_Order
    31     Code_Integer
       
    32     Efficient_Nat
       
    33     (* Code_Prolog  FIXME cf. 76965c356d2a *)
    31     (* Code_Prolog  FIXME cf. 76965c356d2a *)
    34     Code_Real_Approx_By_Float
    32     Code_Real_Approx_By_Float
    35     Code_Target_Numeral
    33     Code_Target_Numeral
    36     IArray
    34     IArray
    37     Refute
    35     Refute
   280   description {* *}
   278   description {* *}
   281   options [document_graph, print_mode = "iff,no_brackets"]
   279   options [document_graph, print_mode = "iff,no_brackets"]
   282   theories [document = false]
   280   theories [document = false]
   283     "~~/src/HOL/Library/Countable"
   281     "~~/src/HOL/Library/Countable"
   284     "~~/src/HOL/Library/Monad_Syntax"
   282     "~~/src/HOL/Library/Monad_Syntax"
   285     "~~/src/HOL/Library/Code_Natural"
       
   286     "~~/src/HOL/Library/LaTeXsugar"
   283     "~~/src/HOL/Library/LaTeXsugar"
   287   theories Imperative_HOL_ex
   284   theories Imperative_HOL_ex
   288   files "document/root.bib" "document/root.tex"
   285   files "document/root.bib" "document/root.tex"
   289 
   286 
   290 session "HOL-Decision_Procs" in Decision_Procs = HOL +
   287 session "HOL-Decision_Procs" in Decision_Procs = HOL +
   297 
   294 
   298 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" +
   295 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" +
   299   description {* Examples for program extraction in Higher-Order Logic *}
   296   description {* Examples for program extraction in Higher-Order Logic *}
   300   options [condition = ISABELLE_POLYML, proofs = 2, parallel_proofs = 0]
   297   options [condition = ISABELLE_POLYML, proofs = 2, parallel_proofs = 0]
   301   theories [document = false]
   298   theories [document = false]
   302     "~~/src/HOL/Library/Efficient_Nat"
   299     "~~/src/HOL/Library/Code_Target_Numeral"
   303     "~~/src/HOL/Library/Monad_Syntax"
   300     "~~/src/HOL/Library/Monad_Syntax"
   304     "~~/src/HOL/Number_Theory/Primes"
   301     "~~/src/HOL/Number_Theory/Primes"
   305     "~~/src/HOL/Number_Theory/UniqueFactorization"
   302     "~~/src/HOL/Number_Theory/UniqueFactorization"
   306     "~~/src/HOL/Library/State_Monad"
   303     "~~/src/HOL/Library/State_Monad"
   307   theories
   304   theories
   313   files "document/root.bib" "document/root.tex"
   310   files "document/root.bib" "document/root.tex"
   314 
   311 
   315 session "HOL-Proofs-Lambda" in "Proofs/Lambda" = "HOL-Proofs" +
   312 session "HOL-Proofs-Lambda" in "Proofs/Lambda" = "HOL-Proofs" +
   316   options [document_graph, print_mode = "no_brackets", proofs = 2, parallel_proofs = 0]
   313   options [document_graph, print_mode = "no_brackets", proofs = 2, parallel_proofs = 0]
   317   theories [document = false]
   314   theories [document = false]
   318     "~~/src/HOL/Library/Code_Integer"
   315     "~~/src/HOL/Library/Code_Target_Int"
   319   theories
   316   theories
   320     Eta
   317     Eta
   321     StrongNorm
   318     StrongNorm
   322     Standardization
   319     Standardization
   323     WeakNorm
   320     WeakNorm