nipkow [Wed, 19 Oct 2005 06:46:45 +0200] rev 17906
added 2 lemmas
mengj [Wed, 19 Oct 2005 06:33:24 +0200] rev 17905
Added files in order to use external ATPs as oracles and invoke these ATPs by calling Isabelle methods (currently "vampire" and "eprover").
wenzelm [Tue, 18 Oct 2005 17:59:37 +0200] rev 17904
simplified interfaces proof/proof' etc.: perform ProofHistory.apply(s)/current internally;
wenzelm [Tue, 18 Oct 2005 17:59:36 +0200] rev 17903
tuned error msg;
wenzelm [Tue, 18 Oct 2005 17:59:35 +0200] rev 17902
renamed atomize_rule to atomize_cterm;
wenzelm [Tue, 18 Oct 2005 17:59:34 +0200] rev 17901
ObjectLogic.atomize_cterm;
wenzelm [Tue, 18 Oct 2005 17:59:33 +0200] rev 17900
use simplified Toplevel.proof etc.;
wenzelm [Tue, 18 Oct 2005 17:59:32 +0200] rev 17899
back: Toplevel.actual/skip_proof;
use simplified Toplevel.proof etc.;
wenzelm [Tue, 18 Oct 2005 17:59:31 +0200] rev 17898
renamed set_context to context;
data extend: reset context;
wenzelm [Tue, 18 Oct 2005 17:59:30 +0200] rev 17897
renamed set_context to context;
export theory_context;
clear_ss: inherit_context;
rewrite_aux etc.: theory_context;
wenzelm [Tue, 18 Oct 2005 17:59:29 +0200] rev 17896
functor: no Simplifier argument;
Simplifier.theory_context;
wenzelm [Tue, 18 Oct 2005 17:59:28 +0200] rev 17895
moved helper lemma to HilbertChoice.thy;
use actual ObjectLogic.atomize_cterm;
eliminated obsolete sign_of;
wenzelm [Tue, 18 Oct 2005 17:59:27 +0200] rev 17894
Simplifier.theory_context;
replaced get_const by Sign.the_const_type;
eliminated obsolete sign_of;
wenzelm [Tue, 18 Oct 2005 17:59:26 +0200] rev 17893
added lemma exE_some (from specification_package.ML);
wenzelm [Tue, 18 Oct 2005 17:59:25 +0200] rev 17892
Simplifier.theory_context;