| Sun, 10 Dec 2006 15:30:44 +0100 | wenzelm | extract_case: Name.clean; | file | diff | annotate |
| Thu, 07 Dec 2006 23:16:55 +0100 | wenzelm | reorganized structure Tactic vs. MetaSimplifier; | file | diff | annotate |
| Tue, 05 Dec 2006 00:30:38 +0100 | wenzelm | thm/prf: separate official name vs. additional tags; | file | diff | annotate |
| Wed, 29 Nov 2006 04:11:09 +0100 | wenzelm | simplified Logic.count_prems; | file | diff | annotate |
| Thu, 16 Nov 2006 01:07:25 +0100 | wenzelm | moved some fundamental concepts to General/basics.ML; | file | diff | annotate |
| Wed, 02 Aug 2006 22:26:41 +0200 | wenzelm | normalized Proof.context/method type aliases; | file | diff | annotate |
| Wed, 26 Jul 2006 19:37:41 +0200 | wenzelm | Variable.import(T): result includes fixed types/terms; | file | diff | annotate |
| Tue, 11 Jul 2006 12:17:13 +0200 | wenzelm | Name.internal; | file | diff | annotate |
| Sat, 17 Jun 2006 19:37:59 +0200 | wenzelm | mutual_rule: proper context; | 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:01:01 +0200 | wenzelm | use conjunction stuff from conjunction.ML; | file | diff | annotate |
| Wed, 15 Feb 2006 21:34:55 +0100 | wenzelm | removed distinct, renamed gen_distinct to distinct; | file | diff | annotate |
| Sat, 11 Feb 2006 17:17:47 +0100 | wenzelm | tuned; | file | diff | annotate |
| Thu, 02 Feb 2006 16:31:38 +0100 | wenzelm | consumes: negative argument relative to total number of prems; | file | diff | annotate |
| Fri, 27 Jan 2006 19:03:02 +0100 | wenzelm | moved theorem tags from Drule to PureThy; | file | diff | annotate |
| Sat, 21 Jan 2006 23:02:14 +0100 | wenzelm | simplified type attribute; | file | diff | annotate |
| Sat, 07 Jan 2006 12:26:33 +0100 | wenzelm | support nested cases; | file | diff | annotate |
| Thu, 05 Jan 2006 17:14:08 +0100 | wenzelm | added strict_mutual_rule; | file | diff | annotate |
| Thu, 22 Dec 2005 00:29:09 +0100 | wenzelm | consume: expand defs in prems of concls; | file | diff | annotate |
| Thu, 08 Dec 2005 20:16:10 +0100 | wenzelm | removed Syntax.deskolem; | file | diff | annotate |
| Fri, 25 Nov 2005 18:58:43 +0100 | wenzelm | consume: unfold defs in all major prems; | file | diff | annotate |
| Wed, 23 Nov 2005 18:52:04 +0100 | wenzelm | consume: proper treatment of defs; | file | diff | annotate |
| Tue, 22 Nov 2005 19:34:50 +0100 | wenzelm | added type cases/cases_tactic, and CASES, SUBGOAL_CASES; | file | diff | annotate |
| Wed, 16 Nov 2005 17:45:34 +0100 | wenzelm | added THEN_ALL_NEW_CASES; | file | diff | annotate |
| Mon, 31 Oct 2005 16:00:15 +0100 | haftmann | fold_index replacing foldln | file | diff | annotate |
| Sat, 15 Oct 2005 00:08:10 +0200 | wenzelm | export strip_params; | file | diff | annotate |
| Tue, 13 Sep 2005 22:19:46 +0200 | wenzelm | added simple; | file | diff | annotate |
| Mon, 29 Aug 2005 16:18:04 +0200 | wenzelm | use AList operations; | file | diff | annotate |
| Sun, 28 Aug 2005 16:04:51 +0200 | wenzelm | unskolem local vars; | file | diff | annotate |
| Thu, 18 Aug 2005 11:17:48 +0200 | wenzelm | added NO_CASES; | file | diff | annotate |
| Tue, 14 Jun 2005 21:56:55 +0200 | wenzelm | added type tactic; | file | diff | annotate |
| Tue, 31 May 2005 11:53:39 +0200 | wenzelm | make: T option -- actually remove undefined cases; | file | diff | annotate |
| Tue, 17 May 2005 10:19:44 +0200 | wenzelm | tuned; | file | diff | annotate |
| Fri, 04 Mar 2005 15:07:34 +0100 | skalberg | Removed practically all references to Library.foldr. | file | diff | annotate |
| Thu, 03 Mar 2005 12:43:01 +0100 | skalberg | Move towards standard functions. | file | diff | annotate |
| Sun, 13 Feb 2005 17:15:14 +0100 | skalberg | Deleted Library.option type. | file | diff | annotate |
| Mon, 21 Jun 2004 10:25:57 +0200 | kleing | Merged in license change from Isabelle2004 | file | diff | annotate |
| Sat, 21 Feb 2004 08:43:08 +0100 | nipkow | Transitive_Closure: added consumes and case_names attributes | file | diff | annotate |
| Mon, 21 Oct 2002 17:17:40 +0200 | berghofe | Removed Logic.skip_flexpairs. | file | diff | annotate |
| Mon, 07 Oct 2002 19:01:51 +0200 | nipkow | take/drop -> splitAt | file | diff | annotate |
| Mon, 30 Sep 2002 15:44:21 +0200 | nipkow | modified induct method | file | diff | annotate |
| Fri, 26 Jul 2002 21:09:39 +0200 | wenzelm | support for split assumptions in cases (hyps vs. prems); | file | diff | annotate |
| Thu, 17 Jan 2002 21:07:00 +0100 | wenzelm | RuleCases.make interface based on term instead of thm; | file | diff | annotate |
| Tue, 15 Jan 2002 00:13:20 +0100 | wenzelm | save: be slightly more about absent tags; | file | diff | annotate |
| Mon, 12 Nov 2001 23:28:15 +0100 | wenzelm | added empty; | file | diff | annotate |
| Wed, 31 Oct 2001 01:22:27 +0100 | wenzelm | put_consumes: really overwrite existing tag; | file | diff | annotate |
| Tue, 30 Oct 2001 17:29:43 +0100 | wenzelm | removed obsolete make_raw; | file | diff | annotate |
| Sun, 14 Oct 2001 20:09:19 +0200 | wenzelm | use ObjectLogic; | file | diff | annotate |
| Tue, 30 Jan 2001 18:53:46 +0100 | oheimb | added foldln | file | diff | annotate |
| Fri, 12 Jan 2001 16:56:20 +0100 | wenzelm | made SML/NJ happy; | file | diff | annotate |
| Thu, 11 Jan 2001 19:38:37 +0100 | wenzelm | make_raw: do not AutoBind.drop_judgment; | file | diff | annotate |
| Tue, 09 Jan 2001 15:17:08 +0100 | wenzelm | avoid renaming of params in cases; | file | diff | annotate |
| Sun, 07 Jan 2001 21:37:40 +0100 | wenzelm | do not AutoBind.drop_judgment; | file | diff | annotate |
| Sat, 06 Jan 2001 21:31:37 +0100 | wenzelm | support ?case binding; | file | diff | annotate |
| Tue, 28 Nov 2000 01:11:12 +0100 | wenzelm | added consumes, consumes_default; | file | diff | annotate |
| Mon, 06 Nov 2000 22:54:13 +0100 | wenzelm | make: open_parms argument; | file | diff | annotate |
| Thu, 13 Jul 2000 11:36:57 +0200 | wenzelm | make: opaq flag; | file | diff | annotate |
| Fri, 05 May 2000 22:09:41 +0200 | wenzelm | GPLed; | file | diff | annotate |
| Fri, 31 Mar 2000 21:56:13 +0200 | wenzelm | params: preserve case names; | file | diff | annotate |
| Fri, 17 Mar 2000 16:29:35 +0100 | wenzelm | fixed untag; | file | diff | annotate |