Wed, 10 Aug 2016 14:50:59 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Sun, 29 May 2016 14:10:48 +0200 |
nipkow |
added subtheory of longest common prefix
|
file |
diff |
annotate
|
Thu, 26 May 2016 09:05:00 +0200 |
nipkow |
added function "prefixes" and some lemmas
|
file |
diff |
annotate
|
Wed, 25 May 2016 17:40:56 +0200 |
nipkow |
renamed suffix(eq)
|
file |
diff |
annotate
|
Mon, 23 May 2016 22:43:11 +0200 |
nipkow |
renamed prefix* in Library/Sublist
|
file |
diff |
annotate
|
Tue, 01 Sep 2015 22:32:58 +0200 |
wenzelm |
eliminated \<Colon>;
|
file |
diff |
annotate
|
Mon, 06 Jul 2015 22:57:34 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Wed, 17 Jun 2015 11:03:05 +0200 |
wenzelm |
isabelle update_cartouches;
|
file |
diff |
annotate
|
Fri, 10 Apr 2015 11:52:55 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Sun, 02 Nov 2014 17:20:45 +0100 |
wenzelm |
modernized header;
|
file |
diff |
annotate
|
Thu, 03 Jul 2014 09:55:16 +0200 |
Christian Sternagel |
weaker assumption for "list_emb_trans"; added lemma
|
file |
diff |
annotate
|
Thu, 03 Jul 2014 09:55:15 +0200 |
Christian Sternagel |
added monotonicity lemma for list embedding
|
file |
diff |
annotate
|
Thu, 03 Jul 2014 09:55:15 +0200 |
Christian Sternagel |
no built-in reflexivity of list embedding (which is more standard; now embedding is reflexive whenever the base-order is)
|
file |
diff |
annotate
|
Thu, 03 Jul 2014 09:55:15 +0200 |
Christian Sternagel |
renamed "list_hembeq" into slightly shorter "list_emb"
|
file |
diff |
annotate
|
Wed, 19 Feb 2014 10:30:21 +0100 |
traytel |
reverted ba7392b52a7c: List_Prefix not needed anymore by codatatypes
|
file |
diff |
annotate
|
Wed, 20 Nov 2013 18:58:00 +0100 |
blanchet |
factor 'List_Prefix' out of 'Sublist' and move to 'Main' (needed for codatatypes)
|
file |
diff |
annotate
|
Tue, 19 Nov 2013 01:29:50 +0100 |
blanchet |
optimized more bad apples
|
file |
diff |
annotate
|
Tue, 13 Aug 2013 16:25:47 +0200 |
wenzelm |
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
|
file |
diff |
annotate
|
Thu, 25 Jul 2013 08:57:16 +0200 |
haftmann |
factored syntactic type classes for bot and top (by Alessandro Coglio)
|
file |
diff |
annotate
|
Thu, 13 Dec 2012 13:11:38 +0100 |
Christian Sternagel |
renamed "emb" to "list_hembeq";
|
file |
diff |
annotate
|
Mon, 03 Sep 2012 23:03:54 +0200 |
wenzelm |
misc tuning;
|
file |
diff |
annotate
|
Thu, 30 Aug 2012 13:03:03 +0900 |
Christian Sternagel |
List is implicitly imported by Main
|
file |
diff |
annotate
| base
|
Wed, 29 Aug 2012 16:25:35 +0900 |
Christian Sternagel |
introduced "sub" as abbreviation for "emb (op =)";
|
file |
diff |
annotate
| base
|
Wed, 29 Aug 2012 11:05:44 +0900 |
Christian Sternagel |
more lemmas on suffixes and embedding
|
file |
diff |
annotate
| base
|
Wed, 29 Aug 2012 10:57:24 +0900 |
Christian Sternagel |
changed arguement order of suffixeq (to facilitate reading "suffixeq xs ys" as "xs is a (possibly empty) suffix of ys)
|
file |
diff |
annotate
| base
|
Thu, 30 Aug 2012 13:05:11 +0900 |
Christian Sternagel |
added author
|
file |
diff |
annotate
| base
|
Wed, 29 Aug 2012 12:23:14 +0900 |
Christian Sternagel |
dropped ord and bot instance for list prefixes (use locale interpretation instead, which allows users to decide what order to use on lists)
|
file |
diff |
annotate
| base
|
Wed, 29 Aug 2012 10:48:28 +0900 |
Christian Sternagel |
added embedding for lists (constant emb)
|
file |
diff |
annotate
| base
|
Wed, 29 Aug 2012 10:46:11 +0900 |
Christian Sternagel |
renamed (in Sublist): postfix ~> suffixeq, and dropped infix syntax >>=
|
file |
diff |
annotate
| base
|
Wed, 29 Aug 2012 10:35:05 +0900 |
Christian Sternagel |
renamed (in Sublist): prefix ~> prefixeq, strict_prefix ~> prefix
|
file |
diff |
annotate
| base
|
Wed, 29 Aug 2012 10:27:56 +0900 |
Christian Sternagel |
renamed theory List_Prefix into Sublist (since it is not only about prefixes)
|
file |
diff |
annotate
| base
|
Sat, 19 Jul 2008 19:27:13 +0200 |
bulwahn |
added verification framework for the HeapMonad and quicksort as example for this framework
|
file |
diff |
annotate
|