| Thu, 19 Oct 2023 17:06:39 +0200 |
wenzelm |
clarified signature;
|
file |
diff |
annotate
|
| Sat, 03 Jun 2023 22:54:24 +1000 |
nipkow |
TN has enough examples of the bug.
|
file |
diff |
annotate
|
| Tue, 18 Apr 2023 22:24:48 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Wed, 20 Oct 2021 18:13:17 +0200 |
wenzelm |
discontinued obsolete "val extend = I" for data slots;
|
file |
diff |
annotate
|
| Fri, 10 Sep 2021 14:59:19 +0200 |
wenzelm |
clarified signature: more scalable operations;
|
file |
diff |
annotate
|
| Sun, 18 Feb 2018 15:05:21 +0100 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
| Thu, 08 Jun 2017 23:37:01 +0200 |
boehmes |
replace non-arithmetic terms by fresh variables before replaying linear-arithmetic proofs: avoid failed proof replays due to an overambitious simpset which may cause proof replay to diverge from the pre-computed proof trace
|
file |
diff |
annotate
|
| Sat, 04 Jun 2016 16:10:44 +0200 |
wenzelm |
Integer.lcm normalizes the sign as in HOL/GCD.thy;
|
file |
diff |
annotate
|
| Wed, 01 Jun 2016 10:45:35 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
| Sun, 13 Dec 2015 21:56:15 +0100 |
wenzelm |
more general types Proof.method / context_tactic;
|
file |
diff |
annotate
|
| Fri, 25 Sep 2015 20:37:59 +0200 |
wenzelm |
moved remaining display.ML to more_thm.ML;
|
file |
diff |
annotate
|
| Wed, 09 Sep 2015 20:57:21 +0200 |
wenzelm |
simplified simproc programming interfaces;
|
file |
diff |
annotate
|
| Wed, 02 Sep 2015 23:18:39 +0200 |
wenzelm |
trim context for persistent storage;
|
file |
diff |
annotate
|
| Sun, 05 Jul 2015 15:02:30 +0200 |
wenzelm |
simplified Thm.instantiate and derivatives: the LHS refers to non-certified variables -- this merely serves as index into already certified structures (or is ignored);
|
file |
diff |
annotate
|
| Mon, 01 Jun 2015 18:59:20 +0200 |
haftmann |
dropped dead code
|
file |
diff |
annotate
|
| Fri, 10 Apr 2015 11:31:10 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
| Mon, 09 Mar 2015 11:21:00 +0100 |
wenzelm |
eliminated dead code (cf. 5e5c36b051af);
|
file |
diff |
annotate
|
| Fri, 06 Mar 2015 23:56:43 +0100 |
wenzelm |
clarified context;
|
file |
diff |
annotate
|
| Fri, 06 Mar 2015 15:58:56 +0100 |
wenzelm |
Thm.cterm_of and Thm.ctyp_of operate on local context;
|
file |
diff |
annotate
|
| Wed, 04 Mar 2015 22:05:01 +0100 |
wenzelm |
clarified signature;
|
file |
diff |
annotate
|
| Wed, 04 Mar 2015 20:47:29 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Wed, 04 Mar 2015 19:53:18 +0100 |
wenzelm |
tuned signature -- prefer qualified names;
|
file |
diff |
annotate
|
| Tue, 10 Feb 2015 14:48:26 +0100 |
wenzelm |
proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
|
file |
diff |
annotate
|
| Wed, 26 Nov 2014 20:05:34 +0100 |
wenzelm |
renamed "pairself" to "apply2", in accordance to @{apply 2};
|
file |
diff |
annotate
|
| Thu, 30 Oct 2014 22:45:19 +0100 |
wenzelm |
eliminated aliases;
|
file |
diff |
annotate
|
| Sun, 09 Feb 2014 13:07:23 +0100 |
nipkow |
disabled counterexample output for now; confusing because often incorrect
|
file |
diff |
annotate
|
| Fri, 24 May 2013 17:00:46 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
| Sat, 11 May 2013 16:57:18 +0200 |
wenzelm |
prefer explicitly qualified exceptions, which is particular important for robust handlers;
|
file |
diff |
annotate
|
| Thu, 18 Apr 2013 17:07:01 +0200 |
wenzelm |
simplifier uses proper Proof.context instead of historic type simpset;
|
file |
diff |
annotate
|
| Sat, 15 Sep 2012 20:13:25 +0200 |
haftmann |
dropped some unused identifiers
|
file |
diff |
annotate
|
| Wed, 21 Mar 2012 11:00:34 +0100 |
wenzelm |
prefer explicitly qualified exception List.Empty;
|
file |
diff |
annotate
|
| Mon, 27 Feb 2012 16:05:51 +0100 |
wenzelm |
clarified prems_lin_arith_tac, with subtle change of semantics: structured prems are inserted as well;
|
file |
diff |
annotate
|
| Fri, 02 Sep 2011 17:58:32 +0200 |
wenzelm |
proper config option linarith_trace;
|
file |
diff |
annotate
|
| Thu, 30 Jun 2011 16:07:30 +0200 |
wenzelm |
merged
|
file |
diff |
annotate
|
| Wed, 29 Jun 2011 11:58:35 +0200 |
boehmes |
linarith counterexamples now provide only valuations for variables (which should restrict the number of linarith trace messages);
|
file |
diff |
annotate
|
| Wed, 29 Jun 2011 21:34:16 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
| Mon, 27 Jun 2011 13:52:47 +0200 |
blanchet |
clarify warning message to avoid confusing beginners
|
file |
diff |
annotate
|
| Thu, 09 Jun 2011 20:22:22 +0200 |
wenzelm |
tuned signature: Name.invent and Name.invent_names;
|
file |
diff |
annotate
|
| Sat, 16 Apr 2011 16:15:37 +0200 |
wenzelm |
modernized structure Proof_Context;
|
file |
diff |
annotate
|
| Mon, 10 Jan 2011 16:45:28 +0100 |
wenzelm |
added merge_options convenience;
|
file |
diff |
annotate
|
| Wed, 03 Nov 2010 11:06:22 +0100 |
wenzelm |
replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
|
file |
diff |
annotate
|
| Thu, 26 Aug 2010 20:42:09 +0200 |
wenzelm |
Fast_Lin_Arith.number_of: more conventional merge that prefers the left side -- note that former ordering wrt. serial numbers makes it depend on accidental load order;
|
file |
diff |
annotate
|
| Thu, 26 Aug 2010 17:37:26 +0200 |
wenzelm |
slightly more abstract data handling in Fast_Lin_Arith;
|
file |
diff |
annotate
|
| Wed, 28 Jul 2010 14:09:56 +0200 |
haftmann |
dropped dead code
|
file |
diff |
annotate
|
| Sat, 15 May 2010 21:50:05 +0200 |
wenzelm |
less pervasive names from structure Thm;
|
file |
diff |
annotate
|
| Wed, 05 May 2010 18:25:34 +0200 |
haftmann |
farewell to old-style mem infixes -- type inference in situations with mem_int and mem_string should provide enough information to resolve the type of (op =)
|
file |
diff |
annotate
|
| Mon, 22 Mar 2010 11:45:09 +0100 |
boehmes |
removed warning_count (known causes for warnings have been resolved)
|
file |
diff |
annotate
|
| Mon, 22 Mar 2010 09:39:10 +0100 |
boehmes |
removed e-mail address from error message
|
file |
diff |
annotate
|
| Sat, 13 Mar 2010 16:44:12 +0100 |
wenzelm |
removed old CVS Ids;
|
file |
diff |
annotate
|
| Tue, 09 Mar 2010 16:30:43 +0100 |
hoelzl |
Use same order of neq-elimination as in proof search.
|
file |
diff |
annotate
|
| Fri, 19 Feb 2010 11:49:44 +0100 |
wenzelm |
Lin_Arith.pre_tac: inherit proper simplifier context, and get rid of posthoc renaming of bound variables;
|
file |
diff |
annotate
|
| Sun, 08 Nov 2009 16:30:41 +0100 |
wenzelm |
adapted Generic_Data, Proof_Data;
|
file |
diff |
annotate
|
| Thu, 29 Oct 2009 17:58:26 +0100 |
wenzelm |
standardized filter/filter_out;
|
file |
diff |
annotate
|
| Tue, 27 Oct 2009 22:56:14 +0100 |
wenzelm |
eliminated some old folds;
|
file |
diff |
annotate
|
| Wed, 21 Oct 2009 12:02:56 +0200 |
haftmann |
curried union as canonical list operation
|
file |
diff |
annotate
|
| Wed, 21 Oct 2009 08:14:38 +0200 |
haftmann |
dropped redundant gen_ prefix
|
file |
diff |
annotate
|
| Tue, 20 Oct 2009 16:13:01 +0200 |
haftmann |
replaced old_style infixes eq_set, subset, union, inter and variants by generic versions
|
file |
diff |
annotate
|
| Mon, 19 Oct 2009 21:54:57 +0200 |
wenzelm |
uniform use of Integer.add/mult/sum/prod;
|
file |
diff |
annotate
|
| Thu, 15 Oct 2009 23:28:10 +0200 |
wenzelm |
replaced String.concat by implode;
|
file |
diff |
annotate
|
| Tue, 29 Sep 2009 16:24:36 +0200 |
wenzelm |
explicit indication of Unsynchronized.ref;
|
file |
diff |
annotate
|
| Thu, 30 Jul 2009 12:20:43 +0200 |
wenzelm |
qualified Subgoal.FOCUS;
|
file |
diff |
annotate
|
| Sun, 26 Jul 2009 22:24:13 +0200 |
wenzelm |
replaced old METAHYPS by FOCUS;
|
file |
diff |
annotate
|
| Tue, 21 Jul 2009 01:03:18 +0200 |
wenzelm |
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
|
file |
diff |
annotate
|
| Fri, 10 Jul 2009 07:59:27 +0200 |
haftmann |
dropped find_index_eq
|
file |
diff |
annotate
|
| Mon, 15 Jun 2009 09:43:30 +0200 |
haftmann |
made SML/NJ happy
|
file |
diff |
annotate
|
| Tue, 09 Jun 2009 09:22:58 +0200 |
boehmes |
tuned
|
file |
diff |
annotate
|
| Mon, 08 Jun 2009 22:29:37 +0200 |
boehmes |
fast_lin_arith uses proper multiplication instead of unfolding to additions
|
file |
diff |
annotate
|
| Mon, 11 May 2009 15:57:30 +0200 |
haftmann |
mk_number replaces number_of
|
file |
diff |
annotate
|
| Mon, 23 Mar 2009 19:01:16 +0100 |
haftmann |
tuned error messages
|
file |
diff |
annotate
|
| Tue, 10 Mar 2009 08:47:45 +0000 |
webertj |
Instead of giving up entirely, arith now ignores all inequalities when there are too many.
|
file |
diff |
annotate
|
| Thu, 29 May 2008 23:46:41 +0200 |
wenzelm |
added warning_count for issued reconstruction failure messages (limit 10);
|
file |
diff |
annotate
|
| Sun, 18 May 2008 15:04:31 +0200 |
wenzelm |
renamed type decompT to decomp;
|
file |
diff |
annotate
|
| Wed, 07 May 2008 10:59:50 +0200 |
berghofe |
Lookup and union operations on terms are now modulo eta conversion.
|
file |
diff |
annotate
|
| Tue, 09 Oct 2007 00:20:13 +0200 |
wenzelm |
generic Syntax.pretty/string_of operations;
|
file |
diff |
annotate
|
| Tue, 18 Sep 2007 16:08:00 +0200 |
wenzelm |
simplified type int (eliminated IntInf.int, integer);
|
file |
diff |
annotate
|
| Wed, 01 Aug 2007 16:55:40 +0200 |
wenzelm |
simplified internal Config interface;
|
file |
diff |
annotate
|
| Tue, 31 Jul 2007 00:56:29 +0200 |
wenzelm |
arith method setup: proper context;
|
file |
diff |
annotate
|
| Sun, 29 Jul 2007 14:29:54 +0200 |
wenzelm |
renamed Drule.add/del/merge_rules to Thm.add/del/merge_thms;
|
file |
diff |
annotate
|
| Thu, 05 Jul 2007 00:06:14 +0200 |
wenzelm |
avoid polymorphic equality;
|
file |
diff |
annotate
|
| Fri, 29 Jun 2007 21:23:05 +0200 |
haftmann |
tuned arithmetic modules
|
file |
diff |
annotate
|
| Sat, 09 Jun 2007 00:28:46 +0200 |
wenzelm |
simplified type integer;
|
file |
diff |
annotate
|
| Tue, 05 Jun 2007 19:19:30 +0200 |
haftmann |
tuned integers
|
file |
diff |
annotate
|
| Sat, 02 Jun 2007 03:15:35 +0200 |
webertj |
cosmetic
|
file |
diff |
annotate
|
| Fri, 01 Jun 2007 23:52:06 +0200 |
webertj |
additional tracing information
|
file |
diff |
annotate
|
| Fri, 01 Jun 2007 16:04:13 +0200 |
webertj |
fixed handling of meta-logic propositions
|
file |
diff |
annotate
|
| Mon, 21 May 2007 19:11:42 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
| Sat, 19 May 2007 11:33:31 +0200 |
haftmann |
dropped nonsense comment
|
file |
diff |
annotate
|
| Sun, 13 May 2007 18:15:25 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
| Mon, 07 May 2007 00:49:59 +0200 |
wenzelm |
simplified DataFun interfaces;
|
file |
diff |
annotate
|
| Wed, 04 Apr 2007 23:29:33 +0200 |
wenzelm |
rep_thm/cterm/ctyp: removed obsolete sign field;
|
file |
diff |
annotate
|
| Wed, 04 Apr 2007 00:11:03 +0200 |
wenzelm |
removed obsolete sign_of/sign_of_thm;
|
file |
diff |
annotate
|
| Tue, 31 Oct 2006 09:28:52 +0100 |
haftmann |
dropped nth_update
|
file |
diff |
annotate
|
| Wed, 30 Aug 2006 03:30:09 +0200 |
webertj |
lin_arith_prover: splitting reverted because of performance loss
|
file |
diff |
annotate
|
| Wed, 02 Aug 2006 03:33:28 +0200 |
webertj |
type annotations fixed (IntInf.int, to make SML/NJ happy)
|
file |
diff |
annotate
|
| Tue, 01 Aug 2006 14:58:43 +0200 |
webertj |
possible disagreement between proof search and proof reconstruction when eliminating inequalities over different types fixed
|
file |
diff |
annotate
|
| Mon, 31 Jul 2006 15:29:36 +0200 |
webertj |
code reformatted
|
file |
diff |
annotate
|
| Sat, 29 Jul 2006 13:15:12 +0200 |
webertj |
lin_arith_prover splits certain operators (e.g. min, max, abs)
|
file |
diff |
annotate
|
| Wed, 26 Jul 2006 19:23:04 +0200 |
webertj |
linear arithmetic splits certain operators (e.g. min, max, abs)
|
file |
diff |
annotate
|
| Thu, 11 May 2006 19:19:33 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Sat, 29 Apr 2006 23:16:43 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Thu, 27 Apr 2006 15:06:35 +0200 |
wenzelm |
tuned basic list operators (flat, maps, map_filter);
|
file |
diff |
annotate
|
| Fri, 24 Mar 2006 11:54:07 +0100 |
berghofe |
Removed occurrences of makestring, which does not
|
file |
diff |
annotate
|
| Wed, 22 Mar 2006 14:06:29 +0100 |
webertj |
comment fixed
|
file |
diff |
annotate
|
| Wed, 22 Mar 2006 11:54:54 +0100 |
webertj |
comment for conjI added
|
file |
diff |
annotate
|
| Wed, 15 Feb 2006 21:34:59 +0100 |
wenzelm |
counter example: avoid vacuous trace;
|
file |
diff |
annotate
|
| Thu, 19 Jan 2006 21:22:08 +0100 |
wenzelm |
setup: theory -> theory;
|
file |
diff |
annotate
|
| Wed, 04 Jan 2006 16:37:57 +0100 |
nipkow |
removed pointless trace msg.
|
file |
diff |
annotate
|
| Fri, 02 Dec 2005 08:06:59 +0100 |
haftmann |
introduced new map2, fold
|
file |
diff |
annotate
|
| Fri, 28 Oct 2005 16:35:40 +0200 |
haftmann |
cleaned up nth, nth_update, nth_map and nth_string functions
|
file |
diff |
annotate
|
| Fri, 21 Oct 2005 14:49:04 +0200 |
haftmann |
introduced functions from Pure/General/rat.ML
|
file |
diff |
annotate
|
| Tue, 18 Oct 2005 17:59:25 +0200 |
wenzelm |
Simplifier.theory_context;
|
file |
diff |
annotate
|
| Mon, 17 Oct 2005 23:10:15 +0200 |
wenzelm |
Simplifier.inherit_context instead of Simplifier.inherit_bounds;
|
file |
diff |
annotate
|
| Fri, 23 Sep 2005 22:21:53 +0200 |
wenzelm |
Simplifier.inherit_bounds;
|
file |
diff |
annotate
|
| Tue, 20 Sep 2005 18:42:56 +0200 |
paulson |
fixed syntax for sml/nj
|
file |
diff |
annotate
|
| Tue, 20 Sep 2005 14:06:00 +0200 |
wenzelm |
Simplifier.inherit_bounds;
|
file |
diff |
annotate
|
| Tue, 20 Sep 2005 08:21:49 +0200 |
haftmann |
slight adaptions to library changes
|
file |
diff |
annotate
|
| Mon, 12 Sep 2005 18:20:32 +0200 |
haftmann |
introduced new-style AList operations
|
file |
diff |
annotate
|
| Sun, 07 Aug 2005 12:30:45 +0200 |
nipkow |
moved some rat functions to library.ML
|
file |
diff |
annotate
|
| Thu, 07 Jul 2005 12:42:50 +0200 |
nipkow |
takes & in premises apart now.
|
file |
diff |
annotate
|
| Fri, 17 Jun 2005 18:35:27 +0200 |
wenzelm |
accomodate change of TheoryDataFun;
|
file |
diff |
annotate
|