| Wed, 09 Sep 2009 11:31:20 +0200 | 
haftmann | 
moved eq handling in nbe into separate oracle
 | 
file |
diff |
annotate
 | 
| Wed, 26 Aug 2009 11:40:28 +0200 | 
boehmes | 
added further conversions and conversionals
 | 
file |
diff |
annotate
 | 
| Fri, 24 Jul 2009 21:21:45 +0200 | 
wenzelm | 
renamed functor BlastFun to Blast, require explicit theory;
 | 
file |
diff |
annotate
 | 
| Fri, 24 Jul 2009 18:58:58 +0200 | 
wenzelm | 
renamed functor ProjectRuleFun to Project_Rule;
 | 
file |
diff |
annotate
 | 
| Fri, 24 Jul 2009 12:33:00 +0200 | 
wenzelm | 
renamed functor InductFun to Induct;
 | 
file |
diff |
annotate
 | 
| Thu, 23 Jul 2009 18:44:09 +0200 | 
wenzelm | 
renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;
 | 
file |
diff |
annotate
 | 
| Tue, 21 Jul 2009 14:36:26 +0200 | 
haftmann | 
moved abstract algebra section to the end
 | 
file |
diff |
annotate
 | 
| Tue, 14 Jul 2009 16:27:31 +0200 | 
haftmann | 
tuned code annotations
 | 
file |
diff |
annotate
 | 
| Tue, 14 Jul 2009 10:54:04 +0200 | 
haftmann | 
code attributes use common underscore convention
 | 
file |
diff |
annotate
 | 
| Tue, 07 Jul 2009 17:21:26 +0200 | 
haftmann | 
more accurate certificates for constant aliasses
 | 
file |
diff |
annotate
 | 
| Thu, 02 Jul 2009 17:34:14 +0200 | 
wenzelm | 
renamed NamedThmsFun to Named_Thms;
 | 
file |
diff |
annotate
 | 
| Thu, 25 Jun 2009 14:59:29 +0200 | 
haftmann | 
arbitrary farewell
 | 
file |
diff |
annotate
 | 
| Sat, 30 May 2009 12:52:57 +0200 | 
wenzelm | 
modernized method setup;
 | 
file |
diff |
annotate
 | 
| Sat, 16 May 2009 15:24:35 +0200 | 
bulwahn | 
merged
 | 
file |
diff |
annotate
 | 
| Sat, 16 May 2009 15:23:52 +0200 | 
bulwahn | 
added collection of simplification rules of recursive functions for quickcheck
 | 
file |
diff |
annotate
 | 
| Sat, 16 May 2009 11:28:02 +0200 | 
nipkow | 
"{x. P x & x=t & Q x}" is now rewritten to "if P t & Q t then {t} else {}"
 | 
file |
diff |
annotate
 | 
| Thu, 14 May 2009 15:09:48 +0200 | 
haftmann | 
merged module code_unit.ML into code.ML
 | 
file |
diff |
annotate
 | 
| Thu, 14 May 2009 09:16:34 +0200 | 
haftmann | 
rewrite op = == eq handled by simproc
 | 
file |
diff |
annotate
 | 
| Wed, 13 May 2009 18:41:35 +0200 | 
haftmann | 
itself is instance of eq
 | 
file |
diff |
annotate
 | 
| Tue, 12 May 2009 19:30:33 +0200 | 
haftmann | 
transferred code generator preprocessor into separate module
 | 
file |
diff |
annotate
 | 
| Wed, 29 Apr 2009 17:15:01 -0700 | 
huffman | 
reimplement reorientation simproc using theory data
 | 
file |
diff |
annotate
 | 
| Sat, 25 Apr 2009 21:28:04 +0200 | 
wenzelm | 
misc cleanup of auto_solve and quickcheck:
 | 
file |
diff |
annotate
 | 
| Fri, 24 Apr 2009 08:24:54 +0200 | 
haftmann | 
generic postprocessing scheme for term evaluations
 | 
file |
diff |
annotate
 | 
| Thu, 23 Apr 2009 12:17:50 +0200 | 
haftmann | 
avoid local [code]
 | 
file |
diff |
annotate
 | 
| Fri, 17 Apr 2009 14:29:56 +0200 | 
haftmann | 
re-engineering of evaluation conversions
 | 
file |
diff |
annotate
 | 
| Wed, 15 Apr 2009 15:52:37 +0200 | 
haftmann | 
code generator bootstrap theory src/Tools/Code_Generator.thy
 | 
file |
diff |
annotate
 | 
| Wed, 15 Apr 2009 15:34:54 +0200 | 
haftmann | 
wrecked old code_funcgr module
 | 
file |
diff |
annotate
 | 
| Fri, 20 Mar 2009 17:12:37 +0100 | 
wenzelm | 
Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
 | 
file |
diff |
annotate
 | 
| Sat, 07 Mar 2009 17:05:40 +0100 | 
blanchet | 
Removed "nitpick_maybe" constant. Makarius now taught me a much nicer trick.
 | 
file |
diff |
annotate
 | 
| Fri, 06 Mar 2009 15:31:07 +0100 | 
blanchet | 
Added a "nitpick_maybe" symbol, which is used by Nitpick. This will go away once Nitpick is part of HOL.
 | 
file |
diff |
annotate
 | 
| Wed, 04 Mar 2009 18:18:05 +0100 | 
blanchet | 
Second try at adding "nitpick_const_def" attribute.
 | 
file |
diff |
annotate
 | 
| Wed, 04 Mar 2009 11:05:29 +0100 | 
blanchet | 
Merge.
 | 
file |
diff |
annotate
 | 
| Wed, 04 Mar 2009 10:45:52 +0100 | 
blanchet | 
Merge.
 | 
file |
diff |
annotate
 | 
| Sun, 01 Mar 2009 18:40:16 +0100 | 
blanchet | 
Added "nitpick_const_def" attribute, for overriding the definition axiom of a constant.
 | 
file |
diff |
annotate
 | 
| Mon, 02 Mar 2009 16:58:39 +0100 | 
haftmann | 
reduced confusion code_funcgr vs. code_wellsorted
 | 
file |
diff |
annotate
 | 
| Sat, 28 Feb 2009 14:52:21 +0100 | 
wenzelm | 
moved generic intuitionistic prover to src/Tools/intuitionistic.ML;
 | 
file |
diff |
annotate
 | 
| Sat, 28 Feb 2009 14:02:12 +0100 | 
wenzelm | 
moved some generic tools to src/Tools/ -- src/Provers is essentially obsolete;
 | 
file |
diff |
annotate
 | 
| Sun, 22 Feb 2009 22:32:50 +0100 | 
haftmann | 
experimental switch to new well-sorting algorithm
 | 
file |
diff |
annotate
 | 
| Sun, 22 Feb 2009 10:22:29 +0100 | 
haftmann | 
formal dependency on newly emerging algorithm
 | 
file |
diff |
annotate
 | 
| Fri, 20 Feb 2009 14:49:24 +0100 | 
haftmann | 
reverted to old wellsorting algorithm
 | 
file |
diff |
annotate
 | 
| Fri, 20 Feb 2009 10:14:31 +0100 | 
haftmann | 
experimental inclusion of new wellsorting algorithm for code equations
 | 
file |
diff |
annotate
 | 
| Wed, 18 Feb 2009 19:18:31 +0100 | 
haftmann | 
do not drop arguments to 0, 1
 | 
file |
diff |
annotate
 | 
| Tue, 10 Feb 2009 14:02:45 +0100 | 
blanchet | 
Renamed descriptions of Nitpick (and ATP) attributes, so that they fit well with the rest of the sentence in ProofGeneral.
 | 
file |
diff |
annotate
 | 
| Mon, 09 Feb 2009 12:31:36 +0100 | 
blanchet | 
Reintroduced nitpick_ind_intro attribute.
 | 
file |
diff |
annotate
 | 
| Mon, 09 Feb 2009 10:37:59 +0100 | 
blanchet | 
Added Nitpick_Const_Psimp attribute, dropped the 's' in Nitpick_Const_Simps, and killed the Nitpick_Ind_Intros attribute.
 | 
file |
diff |
annotate
 | 
| Fri, 06 Feb 2009 15:57:47 +0100 | 
blanchet | 
Added "nitpick_const_simps" and "nitpick_ind_intros" attributes for theorems;
 | 
file |
diff |
annotate
 | 
| Wed, 21 Jan 2009 23:40:23 +0100 | 
haftmann | 
no base sort in class import
 | 
file |
diff |
annotate
 | 
| Fri, 16 Jan 2009 08:29:11 +0100 | 
haftmann | 
added HOL-Base image
 | 
file |
diff |
annotate
 | 
| Mon, 15 Dec 2008 09:58:45 +0100 | 
haftmann | 
moved value.ML to src/Tools
 | 
file |
diff |
annotate
 | 
| Wed, 03 Dec 2008 15:58:44 +0100 | 
haftmann | 
made repository layout more coherent with logical distribution structure; stripped some $Id$s
 | 
file |
diff |
annotate
 | 
| Thu, 20 Nov 2008 00:03:47 +0100 | 
wenzelm | 
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 | 
file |
diff |
annotate
 | 
| Thu, 13 Nov 2008 15:58:38 +0100 | 
haftmann | 
simproc for let
 | 
file |
diff |
annotate
 | 
| Tue, 28 Oct 2008 11:03:07 +0100 | 
ballarin | 
Removed 'includes meta_term_syntax' and 'includes meta_conjunction_syntax'.
 | 
file |
diff |
annotate
 | 
| Fri, 24 Oct 2008 17:48:34 +0200 | 
haftmann | 
"arbitrary" merely abbreviates undefined
 | 
file |
diff |
annotate
 | 
| Wed, 22 Oct 2008 14:15:45 +0200 | 
haftmann | 
code identifier namings are no longer imperative
 | 
file |
diff |
annotate
 | 
| Fri, 10 Oct 2008 06:45:53 +0200 | 
haftmann | 
`code func` now just `code`
 | 
file |
diff |
annotate
 | 
| Tue, 07 Oct 2008 16:07:16 +0200 | 
haftmann | 
re-introduces axiom subst
 | 
file |
diff |
annotate
 | 
| Mon, 29 Sep 2008 12:31:57 +0200 | 
haftmann | 
polished code generator setup
 | 
file |
diff |
annotate
 | 
| Thu, 25 Sep 2008 09:28:03 +0200 | 
haftmann | 
discontinued special treatment of op = vs. eq_class.eq
 | 
file |
diff |
annotate
 | 
| Mon, 22 Sep 2008 23:00:15 +0200 | 
berghofe | 
Added setup for coherent logic prover.
 | 
file |
diff |
annotate
 |