src/HOL/ex/ROOT.ML
author wenzelm
Tue, 06 Jan 2009 21:55:51 +0100
changeset 29376 2071939cf0fc
parent 29181 cc177742e607
child 29377 e6439dbfeee1
permissions -rw-r--r--
more parallel loading;

(*  Title:      HOL/ex/ROOT.ML

Miscellaneous examples for Higher-Order Logic.
*)

no_document use_thys [
  "State_Monad",
  "Efficient_Nat_examples",
  "ExecutableContent",
  "FuncSet",
  "Word",
  "Eval_Examples",
  "Quickcheck",
  "Term_Of_Syntax",
  "Codegenerator",
  "Codegenerator_Pretty",
  "NormalForm"
];

use_thys [
  "Numeral",
  "ImperativeQuicksort",
  "Higher_Order_Logic",
  "Abstract_NAT",
  "Guess",
  "Binary",
  "Recdefs",
  "Fundefs",
  "Induction_Scheme",
  "InductiveInvariant_examples",
  "LocaleTest2",
  "Records",
  "MonoidGroup",
  "BinEx",
  "Hex_Bin_Examples",
  "Antiquote",
  "Multiquote",
  "PER",
  "NatSum",
  "ThreeDivides",
  "Intuitionistic",
  "CTL",
  "Arith_Examples",
  "BT",
  "MergeSort",
  "Lagrange",
  "Groebner_Examples",
  "MT",
  "Unification",
  "Commutative_RingEx",
  "Commutative_Ring_Complete",
  "Primrec",
  "Tarski",
  "Adder",
  "Classical",
  "set",
  "Meson_Test",
  "Code_Antiq",
  "Termination",
  "Coherent",
  "Dense_Linear_Order_Ex",
  "PresburgerEx",
  "Reflected_Presburger",
  "Reflection",
  "ReflectionEx"
];

setmp Proofterm.proofs 2 use_thy "Hilbert_Classical";


use_thy "SVC_Oracle";

fun svc_enabled () = getenv "SVC_HOME" <> "";
fun if_svc_enabled f x = if svc_enabled () then f x else ();

if_svc_enabled time_use_thy "svc_test";


(* requires a proof-generating SAT solver (zChaff or MiniSAT) to be *)
(* installed:                                                       *)
try use_thy "SAT_Examples";

(* requires zChaff (or some other reasonably fast SAT solver) to be *)
(* installed:                                                       *)
if getenv "ZCHAFF_HOME" <> "" then
  use_thy "Sudoku"
else ();

time_use_thy "Refute_Examples";
time_use_thy "Quickcheck_Examples";

HTML.with_charset "utf-8" (no_document use_thys) ["Hebrew", "Chinese"];

no_document use_thys [
  "../NumberTheory/Factorization",
  "../Library/BigO"
];

use_thys [
  "BinEx",
  "Sqrt",
  "Sqrt_Script",
  "BigO_Complex",

  "Arithmetic_Series_Complex",
  "HarmonicSeries",

  "MIR",
  "ReflectedFerrack"
];