src/HOL/Isar_examples/ROOT.ML
author wenzelm
Tue, 04 Aug 2009 15:59:57 +0200
changeset 32323 8185d3bfcbf1
parent 31758 3edd5f813f01
child 32479 521cc9bf2958
permissions -rw-r--r--
tuned "Bootstrapping the environment"; added "Additional components";

(*  Title:      HOL/Isar_examples/ROOT.ML
    Author:     Markus Wenzel, TU Muenchen

Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
*)

no_document use_thys ["../NumberTheory/Primes", "../NumberTheory/Fibonacci"];

use_thys [
  "Basic_Logic",
  "Cantor",
  "Peirce",
  "Drinker",
  "Expr_Compiler",
  "Group",
  "Summation",
  "Knaster_Tarski",
  "Mutilated_Checkerboard",
  "Puzzle",
  "Nested_Datatype",
  "Hoare_Ex"
];