Sat, 27 Mar 2010 15:20:31 +0100 |
wenzelm |
moved Drule.forall_intr_frees to Thm.forall_intr_frees (in more_thm.ML, which is loaded before pure_thy.ML);
|
file |
diff |
annotate
|
Mon, 22 Mar 2010 19:29:11 +0100 |
wenzelm |
eliminated old-style Drule.add_axiom in favour of Specification.axiom, with explicit Drule.export_without_context to imitate the old behaviour;
|
file |
diff |
annotate
|
Mon, 22 Mar 2010 00:48:56 +0100 |
wenzelm |
replaced PureThy.add_axioms by more basic Drule.add_axiom, which is old-style nonetheless;
|
file |
diff |
annotate
|
Sat, 20 Mar 2010 17:33:11 +0100 |
wenzelm |
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
|
file |
diff |
annotate
|
Fri, 19 Feb 2010 20:39:48 +0100 |
wenzelm |
moved ancient Drule.get_def to OldGoals.get_def;
|
file |
diff |
annotate
|
Sun, 07 Feb 2010 19:33:34 +0100 |
wenzelm |
renamed old-style Drule.standard to Drule.export_without_context, to emphasize that this is in no way a standard operation;
|
file |
diff |
annotate
|
Sat, 21 Nov 2009 15:49:29 +0100 |
wenzelm |
explicitly mark some legacy freeze operations;
|
file |
diff |
annotate
|
Thu, 12 Nov 2009 22:02:11 +0100 |
wenzelm |
eliminated obsolete "internal" kind -- collapsed to unspecific "";
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 20:34:59 +0100 |
wenzelm |
modernized structure Simple_Syntax;
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 16:25:26 +0100 |
wenzelm |
Drule.store: proper binding;
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 19:47:37 +0200 |
wenzelm |
renamed NameSpace to Name_Space -- also to emphasize its subtle change in semantics;
|
file |
diff |
annotate
|
Sat, 17 Oct 2009 00:53:18 +0200 |
wenzelm |
legacy Drule.standard is no longer pervasive;
|
file |
diff |
annotate
|
Thu, 09 Jul 2009 22:48:12 +0200 |
wenzelm |
renamed structure TermSubst to Term_Subst;
|
file |
diff |
annotate
|
Mon, 06 Jul 2009 21:24:30 +0200 |
wenzelm |
structure Thm: less pervasive names;
|
file |
diff |
annotate
|
Thu, 02 Jul 2009 21:26:18 +0200 |
wenzelm |
renamed Drule.sort_triv to Thm.sort_triv (cf. more_thm.ML);
|
file |
diff |
annotate
|
Mon, 16 Mar 2009 23:39:44 +0100 |
wenzelm |
refined is_norm_hhf: reject beta-redexes (rules based on term nets or could_unify assume normal form), also potentially faster by avoiding expensive Envir.beta_eta_contract;
|
file |
diff |
annotate
|
Sat, 07 Mar 2009 22:04:59 +0100 |
wenzelm |
moved Thm.def_name(_optional) to more_thm.ML;
|
file |
diff |
annotate
|
Wed, 21 Jan 2009 16:47:04 +0100 |
haftmann |
binding replaces bstring
|
file |
diff |
annotate
|
Sun, 04 Jan 2009 15:28:09 +0100 |
wenzelm |
added comp_no_flatten;
|
file |
diff |
annotate
|
Wed, 31 Dec 2008 18:53:16 +0100 |
wenzelm |
moved old add_type_XXX, add_term_XXX etc. to structure OldTerm;
|
file |
diff |
annotate
|
Wed, 31 Dec 2008 00:08:13 +0100 |
wenzelm |
moved old add_term_vars, add_term_frees etc. to structure OldTerm;
|
file |
diff |
annotate
|
Fri, 31 Oct 2008 10:39:04 +0100 |
berghofe |
Theorem "_" is now stored with open derivation.
|
file |
diff |
annotate
|
Thu, 23 Oct 2008 15:28:01 +0200 |
wenzelm |
renamed Thm.get_axiom_i to Thm.axiom;
|
file |
diff |
annotate
|
Thu, 16 Oct 2008 22:44:27 +0200 |
wenzelm |
added rules for sort_constraint, include in norm_hhf_eqs;
|
file |
diff |
annotate
|
Thu, 14 Aug 2008 16:52:46 +0200 |
wenzelm |
moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);
|
file |
diff |
annotate
|
Mon, 23 Jun 2008 23:45:46 +0200 |
wenzelm |
Logic.implies;
|
file |
diff |
annotate
|
Thu, 19 Jun 2008 20:48:03 +0200 |
wenzelm |
moved add_used to Isar/rule_insts.ML;
|
file |
diff |
annotate
|
Mon, 16 Jun 2008 22:13:47 +0200 |
wenzelm |
removed obsolete global read_insts/read_instantiate (cf. Isar/rule_insts.ML);
|
file |
diff |
annotate
|
Wed, 11 Jun 2008 18:03:14 +0200 |
wenzelm |
qualified types_sorts, read_insts etc.;
|
file |
diff |
annotate
|
Sun, 18 May 2008 15:04:09 +0200 |
wenzelm |
moved global pretty/string_of functions from Sign to Syntax;
|
file |
diff |
annotate
|
Tue, 15 Apr 2008 16:12:05 +0200 |
wenzelm |
Thm.forall_elim_var(s);
|
file |
diff |
annotate
|
Sat, 12 Apr 2008 17:00:38 +0200 |
wenzelm |
rep_cterm/rep_thm: no longer dereference theory_ref;
|
file |
diff |
annotate
|
Sat, 29 Mar 2008 19:14:09 +0100 |
wenzelm |
certify wrt. dynamic context;
|
file |
diff |
annotate
|
Thu, 27 Mar 2008 14:41:09 +0100 |
wenzelm |
eliminated theory ProtoPure;
|
file |
diff |
annotate
|
Tue, 27 Nov 2007 15:43:31 +0100 |
berghofe |
Better error messages for cterm_instantiate.
|
file |
diff |
annotate
|
Thu, 11 Oct 2007 19:10:20 +0200 |
wenzelm |
moved Drule.unvarify to Thm.unvarify (cf. more_thm.ML);
|
file |
diff |
annotate
|
Wed, 10 Oct 2007 17:31:54 +0200 |
wenzelm |
improved abs_def: only abstract over outermost (unique) Vars;
|
file |
diff |
annotate
|
Thu, 04 Oct 2007 20:29:24 +0200 |
wenzelm |
replaced literal 'a by Name.aT;
|
file |
diff |
annotate
|
Fri, 24 Aug 2007 14:17:54 +0200 |
paulson |
new derived rule: incr_type_indexes
|
file |
diff |
annotate
|
Mon, 13 Aug 2007 18:10:18 +0200 |
wenzelm |
SimpleSyntax.read_prop;
|
file |
diff |
annotate
|
Sun, 29 Jul 2007 14:30:04 +0200 |
wenzelm |
moved Drule.add/del/merge_rules to Thm.add/del/merge_thms;
|
file |
diff |
annotate
|
Fri, 27 Jul 2007 20:11:48 +0200 |
wenzelm |
added dummy_thm, is_dummy_thm;
|
file |
diff |
annotate
|
Wed, 04 Jul 2007 16:49:36 +0200 |
wenzelm |
added binop_cong_rule;
|
file |
diff |
annotate
|
Tue, 03 Jul 2007 17:17:11 +0200 |
wenzelm |
tuned rotate_prems;
|
file |
diff |
annotate
|
Wed, 20 Jun 2007 17:32:53 +0200 |
paulson |
A more robust flexflex_unique
|
file |
diff |
annotate
|
Tue, 19 Jun 2007 23:15:51 +0200 |
wenzelm |
added with_subgoal;
|
file |
diff |
annotate
|
Thu, 31 May 2007 23:47:36 +0200 |
wenzelm |
simplified/unified list fold;
|
file |
diff |
annotate
|
Fri, 11 May 2007 18:49:15 +0200 |
wenzelm |
proper type for fun/arg_cong_rule;
|
file |
diff |
annotate
|
Fri, 11 May 2007 18:47:08 +0200 |
wenzelm |
added fun/arg_cong_rule;
|
file |
diff |
annotate
|
Thu, 10 May 2007 00:39:52 +0200 |
wenzelm |
moved some operations to more_thm.ML and conv.ML;
|
file |
diff |
annotate
|
Sun, 15 Apr 2007 14:31:53 +0200 |
wenzelm |
moved Drule.plain_prop_of, Drule.fold_terms to more_thm.ML;
|
file |
diff |
annotate
|
Sat, 14 Apr 2007 17:36:09 +0200 |
wenzelm |
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
|
file |
diff |
annotate
|
Mon, 02 Apr 2007 11:31:08 +0200 |
paulson |
optimizing the null instantiation case
|
file |
diff |
annotate
|
Mon, 26 Feb 2007 23:18:24 +0100 |
wenzelm |
moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
|
file |
diff |
annotate
|
Tue, 13 Feb 2007 16:37:14 +0100 |
paulson |
COMP now performs a distinctness check on the multiple results before failing
|
file |
diff |
annotate
|
Sat, 10 Feb 2007 16:43:23 +0100 |
paulson |
Completing the bug fix from the previous update: the result of unifying type
|
file |
diff |
annotate
|
Thu, 08 Feb 2007 18:14:13 +0100 |
paulson |
cterm_instantiate was calling a type instantiation function that works only for matching,
|
file |
diff |
annotate
|
Fri, 19 Jan 2007 22:08:18 +0100 |
wenzelm |
moved inst from drule.ML to old_goals.ML;
|
file |
diff |
annotate
|
Tue, 05 Dec 2006 00:30:38 +0100 |
wenzelm |
thm/prf: separate official name vs. additional tags;
|
file |
diff |
annotate
|
Thu, 30 Nov 2006 14:17:27 +0100 |
wenzelm |
added zero_var_indexes_list;
|
file |
diff |
annotate
|
Wed, 29 Nov 2006 23:33:09 +0100 |
wenzelm |
*** bad commit -- reverted to previous version ***
|
file |
diff |
annotate
|
Wed, 29 Nov 2006 23:28:08 +0100 |
wenzelm |
added INCR_COMP, COMP_INCR;
|
file |
diff |
annotate
|
Wed, 29 Nov 2006 04:11:11 +0100 |
wenzelm |
added INCR_COMP, COMP_INCR;
|
file |
diff |
annotate
|
Tue, 28 Nov 2006 00:35:21 +0100 |
wenzelm |
dest_term: strip_imp_concl;
|
file |
diff |
annotate
|
Fri, 24 Nov 2006 22:05:15 +0100 |
wenzelm |
added cterm_rule;
|
file |
diff |
annotate
|
Tue, 21 Nov 2006 18:07:33 +0100 |
wenzelm |
moved theorem kinds from PureThy to Thm;
|
file |
diff |
annotate
|
Mon, 09 Oct 2006 02:19:56 +0200 |
wenzelm |
added dest_equals_lhs;
|
file |
diff |
annotate
|
Sat, 07 Oct 2006 01:31:09 +0200 |
wenzelm |
added term_rule;
|
file |
diff |
annotate
|
Thu, 05 Oct 2006 10:40:12 +0200 |
paulson |
a few new functions on thms and cterms
|
file |
diff |
annotate
|
Thu, 21 Sep 2006 19:04:55 +0200 |
wenzelm |
added dest_equals_rhs;
|
file |
diff |
annotate
|
Mon, 18 Sep 2006 19:39:07 +0200 |
wenzelm |
Thm.dest_arg;
|
file |
diff |
annotate
|
Tue, 12 Sep 2006 12:12:46 +0200 |
wenzelm |
moved term subst functions to TermSubst;
|
file |
diff |
annotate
|
Thu, 03 Aug 2006 17:30:37 +0200 |
wenzelm |
tuned types_sorts, add_used;
|
file |
diff |
annotate
|
Wed, 02 Aug 2006 22:26:52 +0200 |
wenzelm |
removed obsolete frees/vars_of etc.;
|
file |
diff |
annotate
|
Sun, 30 Jul 2006 21:28:52 +0200 |
wenzelm |
Thm.adjust_maxidx;
|
file |
diff |
annotate
|
Thu, 27 Jul 2006 13:43:05 +0200 |
wenzelm |
removed obsolete equal_abs_elim(_list);
|
file |
diff |
annotate
|
Tue, 11 Jul 2006 12:17:02 +0200 |
wenzelm |
replaced Term.variant(list) by Name.variant(_list);
|
file |
diff |
annotate
|
Tue, 04 Jul 2006 19:49:50 +0200 |
wenzelm |
added generalize;
|
file |
diff |
annotate
|
Sat, 17 Jun 2006 19:37:47 +0200 |
wenzelm |
Term.internal;
|
file |
diff |
annotate
|
Tue, 13 Jun 2006 23:41:44 +0200 |
wenzelm |
removed weak_eq_thm;
|
file |
diff |
annotate
|
Mon, 12 Jun 2006 21:19:00 +0200 |
wenzelm |
tuned Seq/Envir/Unify interfaces;
|
file |
diff |
annotate
|
Sun, 11 Jun 2006 21:59:21 +0200 |
wenzelm |
outer_params: Syntax.dest_internal;
|
file |
diff |
annotate
|
Mon, 05 Jun 2006 21:54:21 +0200 |
wenzelm |
support embedded terms;
|
file |
diff |
annotate
|
Thu, 01 Jun 2006 14:51:37 +0200 |
paulson |
Tiny code cleanup
|
file |
diff |
annotate
|
Fri, 26 May 2006 22:20:05 +0200 |
wenzelm |
forall_intr_list: do not ignore errors;
|
file |
diff |
annotate
|
Mon, 01 May 2006 17:05:11 +0200 |
wenzelm |
added sort_triv;
|
file |
diff |
annotate
|
Sat, 29 Apr 2006 23:16:46 +0200 |
wenzelm |
added unconstrainTs;
|
file |
diff |
annotate
|
Thu, 27 Apr 2006 15:06:35 +0200 |
wenzelm |
tuned basic list operators (flat, maps, map_filter);
|
file |
diff |
annotate
|
Thu, 13 Apr 2006 12:00:59 +0200 |
wenzelm |
added equal_elim_rule2;
|
file |
diff |
annotate
|
Sat, 04 Mar 2006 21:10:07 +0100 |
wenzelm |
added mk_conjunction;
|
file |
diff |
annotate
|
Wed, 22 Feb 2006 22:18:38 +0100 |
wenzelm |
removed rename_indexes_wrt;
|
file |
diff |
annotate
|
Wed, 15 Feb 2006 21:35:02 +0100 |
wenzelm |
added distinct_prems_rl;
|
file |
diff |
annotate
|
Mon, 06 Feb 2006 20:58:54 +0100 |
wenzelm |
Envir.(beta_)eta_contract;
|
file |
diff |
annotate
|
Fri, 03 Feb 2006 23:12:30 +0100 |
wenzelm |
removed add/del_rules;
|
file |
diff |
annotate
|
Sat, 28 Jan 2006 17:28:54 +0100 |
wenzelm |
added equals_cong;
|
file |
diff |
annotate
|
Fri, 27 Jan 2006 19:03:02 +0100 |
wenzelm |
moved theorem tags from Drule to PureThy;
|
file |
diff |
annotate
|
Wed, 25 Jan 2006 00:21:35 +0100 |
wenzelm |
abs_def: improved error;
|
file |
diff |
annotate
|
Sat, 21 Jan 2006 23:02:24 +0100 |
wenzelm |
simplified type attribute;
|
file |
diff |
annotate
|
Tue, 10 Jan 2006 19:33:32 +0100 |
wenzelm |
added declaration_attribute;
|
file |
diff |
annotate
|
Sat, 31 Dec 2005 21:49:43 +0100 |
wenzelm |
tuned forall_intr_vars;
|
file |
diff |
annotate
|
Fri, 23 Dec 2005 15:16:46 +0100 |
wenzelm |
conj_elim_precise: proper treatment of nested conjunctions;
|
file |
diff |
annotate
|
Thu, 22 Dec 2005 00:28:54 +0100 |
wenzelm |
fixed has_internal;
|
file |
diff |
annotate
|
Thu, 08 Dec 2005 20:16:10 +0100 |
wenzelm |
removed Syntax.deskolem;
|
file |
diff |
annotate
|
Fri, 02 Dec 2005 22:54:45 +0100 |
wenzelm |
abs_def: beta/eta contract lhs;
|
file |
diff |
annotate
|
Fri, 25 Nov 2005 18:58:37 +0100 |
wenzelm |
forall_conv: limit prefix;
|
file |
diff |
annotate
|
Tue, 22 Nov 2005 19:34:44 +0100 |
wenzelm |
export map_tags;
|
file |
diff |
annotate
|
Sat, 19 Nov 2005 14:21:03 +0100 |
wenzelm |
removed conj_mono;
|
file |
diff |
annotate
|
Wed, 16 Nov 2005 17:45:25 +0100 |
wenzelm |
added protect_cong, cong_mono_thm;
|
file |
diff |
annotate
|
Wed, 09 Nov 2005 16:26:44 +0100 |
wenzelm |
added fold_terms;
|
file |
diff |
annotate
|
Tue, 08 Nov 2005 10:43:09 +0100 |
wenzelm |
removed impose_hyps, satisfy_hyps;
|
file |
diff |
annotate
|
Fri, 28 Oct 2005 22:27:52 +0200 |
wenzelm |
added incr_indexes;
|
file |
diff |
annotate
|
Fri, 21 Oct 2005 18:14:44 +0200 |
wenzelm |
renamed triv_goal to goalI, rev_triv_goal to goalD;
|
file |
diff |
annotate
|
Thu, 29 Sep 2005 12:30:30 +0200 |
berghofe |
Optimized and exported flexflex_unique.
|
file |
diff |
annotate
|
Mon, 26 Sep 2005 19:19:14 +0200 |
wenzelm |
moved disambiguate_frees to ProofKernel;
|
file |
diff |
annotate
|
Mon, 26 Sep 2005 02:06:44 +0200 |
obua |
added Drule.disambiguate_frees : thm -> thm
|
file |
diff |
annotate
|
Mon, 12 Sep 2005 18:20:32 +0200 |
haftmann |
introduced new-style AList operations
|
file |
diff |
annotate
|
Wed, 31 Aug 2005 15:46:40 +0200 |
wenzelm |
refer to theory instead of low-level tsig;
|
file |
diff |
annotate
|
Mon, 01 Aug 2005 19:20:37 +0200 |
wenzelm |
replaced atless by term_ord;
|
file |
diff |
annotate
|
Thu, 28 Jul 2005 15:20:06 +0200 |
wenzelm |
tuned gen_all, forall_elim_list, implies_intr_list, standard;
|
file |
diff |
annotate
|
Fri, 15 Jul 2005 15:44:15 +0200 |
wenzelm |
tuned fold on terms;
|
file |
diff |
annotate
|