src/ZF/ROOT.ML
author wenzelm
Sun, 29 Nov 1998 13:16:47 +0100
changeset 5989 9670dae0143d
parent 5529 4a54acae6a15
child 6053 8a1059aa01f0
permissions -rw-r--r--
proof_general_trans (experimental);

(*  Title:      ZF/ROOT
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1993  University of Cambridge

Adds Zermelo-Fraenkel Set Theory to a database containing First-Order Logic.

This theory is the work of Martin Coen, Philippe Noel and Lawrence Paulson.
*)

val banner = "ZF Set Theory (in FOL)";
writeln banner;

eta_contract:=false;

(*For Pure/tactic??  A crude way of adding structure to rules*)
fun CHECK_SOLVED tac st =
    case Seq.pull (tac st) of
        None => error"DO_GOAL: tactic list failed"
      | Some(x,_) => 
                if has_fewer_prems 1 x then
                    Seq.cons(x, Seq.empty)
                else (writeln"DO_GOAL: unsolved goals!!";
                      writeln"Final proof state was ...";
                      print_goals (!goals_limit) x;
                      raise ERROR);

fun DO_GOAL tfs = SELECT_GOAL (CHECK_SOLVED (EVERY1 tfs));

print_depth 1;

(*Add user sections for inductive/datatype definitions*)
use     "$ISABELLE_HOME/src/Pure/section_utils.ML";
use     "thy_syntax.ML";

use_thy "Let";
use_thy "func";
use     "typechk.ML";
use_thy "InfDatatype";
use_thy "List";

(*Integers & binary integer arithmetic*)
cd "Integ";
use_thy "Bin";
cd "..";

(*the all-in-one theory*)
use_thy "Main";

print_depth 8;

Goal "True";  (*leave subgoal package empty*)

val ZF_build_completed = ();    (*indicate successful build*)