Moved theorems Ord_cases_lemma and Ord_cases here from Univ,
strengthening the succ(j) case to include Ord(j). Proved trans_induct3,
le_implies_UN_le_UN, Ord_1, lt_Ord2, le_Ord2.
(* Title: Modal/ex/ROOT
ID: $Id$
Author: Martin Coen
Copyright 1991 University of Cambridge
*)
Modal_build_completed; (*Cause examples to fail if Modal did*)
proof_timing := true;
writeln "\nTheorems of T\n";
fun try s = (writeln s; prove_goal T.thy s (fn _=> [T_Prover.solve_tac 2]));
time_use "ex/Tthms.ML";
writeln "\nTheorems of S4\n";
fun try s = (writeln s; prove_goal S4.thy s (fn _=> [S4_Prover.solve_tac 2]));
time_use "ex/Tthms.ML";
time_use "ex/S4thms.ML";
writeln "\nTheorems of S43\n";
fun try s = (writeln s;
prove_goal S43.thy s (fn _=> [S43_Prover.solve_tac 2 ORELSE
S43_Prover.solve_tac 3]));
time_use "ex/Tthms.ML";
time_use "ex/S4thms.ML";
time_use "ex/S43thms.ML";
maketest"END: Root file for Modal examples";