Tue, 19 Oct 2004 18:18:45 +0200 |
paulson |
converted some induct_tac to induct
|
file |
diff |
annotate
|
Fri, 15 Oct 2004 18:16:03 +0200 |
nipkow |
added and renamed
|
file |
diff |
annotate
|
Thu, 14 Oct 2004 12:18:52 +0200 |
nipkow |
Added a few lemmas
|
file |
diff |
annotate
|
Mon, 11 Oct 2004 07:42:22 +0200 |
nipkow |
Proofs needed to be updated because induction now preserves name of
|
file |
diff |
annotate
|
Fri, 03 Sep 2004 10:26:39 +0200 |
paulson |
listrel operator for lifting relations to lists
|
file |
diff |
annotate
|
Wed, 01 Sep 2004 15:03:41 +0200 |
paulson |
new functions for sets of lists
|
file |
diff |
annotate
|
Wed, 18 Aug 2004 11:09:40 +0200 |
nipkow |
import -> imports
|
file |
diff |
annotate
|
Mon, 16 Aug 2004 14:22:27 +0200 |
nipkow |
New theory header syntax.
|
file |
diff |
annotate
|
Thu, 05 Aug 2004 10:50:58 +0200 |
paulson |
some structured proofs
|
file |
diff |
annotate
|
Wed, 04 Aug 2004 19:10:45 +0200 |
nipkow |
Added a number of new thms and the new function remove1
|
file |
diff |
annotate
|
Thu, 22 Jul 2004 10:33:26 +0200 |
paulson |
new material courtesy of Norbert Voelker
|
file |
diff |
annotate
|
Mon, 19 Jul 2004 18:19:42 +0200 |
berghofe |
- Moved code generator setup for lists from Main.thy to List.thy
|
file |
diff |
annotate
|
Thu, 15 Jul 2004 13:11:34 +0200 |
nipkow |
Moved to new m<..<n syntax for set intervals.
|
file |
diff |
annotate
|
Mon, 21 Jun 2004 10:25:57 +0200 |
kleing |
Merged in license change from Isabelle2004
|
file |
diff |
annotate
|
Mon, 24 May 2004 18:35:34 +0200 |
nipkow |
added drop_take:thm
|
file |
diff |
annotate
|
Fri, 21 May 2004 21:16:51 +0200 |
wenzelm |
removed duplicate thms;
|
file |
diff |
annotate
|
Fri, 16 Apr 2004 15:46:50 +0200 |
mehta |
lemma drop_Suc_conv_tl added.
|
file |
diff |
annotate
|
Fri, 16 Apr 2004 13:51:04 +0200 |
wenzelm |
tuned document;
|
file |
diff |
annotate
|
Wed, 14 Apr 2004 14:13:05 +0200 |
kleing |
use more symbols in HTML output
|
file |
diff |
annotate
|
Mon, 12 Apr 2004 19:54:32 +0200 |
oheimb |
removed o2l and fold_rel; moved postfix to Library/List_Prefix.thy
|
file |
diff |
annotate
|
Tue, 30 Mar 2004 08:45:39 +0200 |
nipkow |
Added append_eq_append_conv2
|
file |
diff |
annotate
|
Fri, 20 Feb 2004 01:32:59 +0100 |
nipkow |
moved lemmas from MicroJava/Comp/AuxLemmas.thy to List.thy
|
file |
diff |
annotate
|
Thu, 19 Feb 2004 10:40:28 +0100 |
paulson |
new theorem
|
file |
diff |
annotate
|
Mon, 16 Feb 2004 03:25:52 +0100 |
kleing |
lemmas about card (set xs)
|
file |
diff |
annotate
|
Wed, 07 Jan 2004 07:52:12 +0100 |
kleing |
map_idI
|
file |
diff |
annotate
|
Mon, 05 Jan 2004 23:10:32 +0100 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Mon, 05 Jan 2004 22:43:03 +0100 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Wed, 24 Dec 2003 08:54:30 +0100 |
kleing |
list_all2_nthD no good as [intro?]
|
file |
diff |
annotate
|
Tue, 23 Dec 2003 23:40:16 +0100 |
kleing |
list_all2_mono should not be [trans]
|
file |
diff |
annotate
|
Tue, 23 Dec 2003 06:35:41 +0100 |
kleing |
added some [intro?] and [trans] for list_all2 lemmas
|
file |
diff |
annotate
|
Fri, 19 Dec 2003 04:28:45 +0100 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Thu, 18 Dec 2003 08:20:36 +0100 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Wed, 29 Oct 2003 01:17:06 +0100 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Fri, 26 Sep 2003 10:34:57 +0200 |
paulson |
misc tidying
|
file |
diff |
annotate
|
Sun, 14 Sep 2003 17:53:27 +0200 |
nipkow |
Added new theorems
|
file |
diff |
annotate
|
Tue, 15 Jul 2003 08:25:20 +0200 |
nipkow |
Some new thm (ex_map_conv?)
|
file |
diff |
annotate
|
Fri, 11 Jul 2003 14:12:02 +0200 |
oheimb |
added fold_red, o2l, postfix, some thms
|
file |
diff |
annotate
|
Wed, 28 May 2003 10:47:54 +0200 |
paulson |
new theorem
|
file |
diff |
annotate
|
Wed, 14 May 2003 10:22:09 +0200 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Wed, 16 Apr 2003 22:14:08 +0200 |
nipkow |
Added take/dropWhile thms
|
file |
diff |
annotate
|
Tue, 25 Mar 2003 09:58:51 +0100 |
berghofe |
Re-structured some proofs in order to get rid of rule_format attribute.
|
file |
diff |
annotate
|
Fri, 14 Mar 2003 12:03:23 +0100 |
kleing |
more about list_all2
|
file |
diff |
annotate
|
Fri, 29 Nov 2002 09:48:28 +0100 |
nipkow |
added a few lemmas
|
file |
diff |
annotate
|
Mon, 30 Sep 2002 16:14:02 +0200 |
berghofe |
Adapted to new simplifier.
|
file |
diff |
annotate
|
Thu, 26 Sep 2002 10:51:29 +0200 |
paulson |
Converted Fun to Isar style.
|
file |
diff |
annotate
|
Wed, 21 Aug 2002 15:53:30 +0200 |
paulson |
Frederic Blanqui's new "guard" examples
|
file |
diff |
annotate
|
Thu, 08 Aug 2002 23:46:09 +0200 |
wenzelm |
use Tactic.prove instead of prove_goalw_cterm in internal proofs!
|
file |
diff |
annotate
|
Tue, 06 Aug 2002 11:22:05 +0200 |
wenzelm |
sane interface for simprocs;
|
file |
diff |
annotate
|
Tue, 16 Jul 2002 18:26:36 +0200 |
wenzelm |
moved stuff from Main.thy;
|
file |
diff |
annotate
|
Thu, 30 May 2002 10:12:52 +0200 |
nipkow |
Modifications due to enhanced linear arithmetic.
|
file |
diff |
annotate
|
Mon, 13 May 2002 15:45:21 +0200 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Mon, 13 May 2002 15:39:56 +0200 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Mon, 13 May 2002 15:27:28 +0200 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Mon, 13 May 2002 11:05:27 +0200 |
wenzelm |
tuned document;
|
file |
diff |
annotate
|
Wed, 08 May 2002 13:01:40 +0200 |
nipkow |
new thm distinct_conv_nth
|
file |
diff |
annotate
|
Wed, 08 May 2002 12:15:30 +0200 |
wenzelm |
oops;
|
file |
diff |
annotate
|
Tue, 07 May 2002 19:54:29 +0200 |
wenzelm |
converted;
|
file |
diff |
annotate
|
Thu, 14 Feb 2002 11:50:52 +0100 |
nipkow |
nodups -> distinct
|
file |
diff |
annotate
|
Fri, 09 Nov 2001 00:09:47 +0100 |
wenzelm |
eliminated old "symbols" syntax, use "xsymbols" instead;
|
file |
diff |
annotate
|
Tue, 09 Jan 2001 15:22:13 +0100 |
nipkow |
`` -> and ``` -> ``
|
file |
diff |
annotate
|