Tue, 08 Oct 2024 12:10:35 +0200 |
wenzelm |
more inner-syntax markup;
|
file |
diff |
annotate
|
Mon, 23 Sep 2024 22:33:37 +0200 |
wenzelm |
proper 'no_syntax' (amending 8e72f55295fd);
|
file |
diff |
annotate
|
Fri, 20 Sep 2024 19:51:08 +0200 |
wenzelm |
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
|
file |
diff |
annotate
|
Wed, 24 Apr 2024 20:56:26 +0100 |
paulson |
More tidying of proofs
|
file |
diff |
annotate
|
Mon, 22 Apr 2024 22:08:28 +0100 |
paulson |
More tidying of Nominal proofs
|
file |
diff |
annotate
|
Sat, 05 Jan 2019 17:24:33 +0100 |
wenzelm |
isabelle update -u control_cartouches;
|
file |
diff |
annotate
|
Tue, 16 Jan 2018 09:30:00 +0100 |
wenzelm |
standardized towards new-style formal comments: isabelle update_comments;
|
file |
diff |
annotate
|
Fri, 18 Aug 2017 20:47:47 +0200 |
wenzelm |
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
|
file |
diff |
annotate
|
Thu, 26 May 2016 17:51:22 +0200 |
wenzelm |
isabelle update_cartouches -c -t;
|
file |
diff |
annotate
|
Mon, 31 Aug 2015 21:01:21 +0200 |
wenzelm |
prefer symbols;
|
file |
diff |
annotate
|
Thu, 11 Sep 2014 18:54:36 +0200 |
blanchet |
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
|
file |
diff |
annotate
|
Wed, 12 Feb 2014 08:37:06 +0100 |
blanchet |
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
|
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
|
Wed, 28 Nov 2012 15:59:18 +0100 |
wenzelm |
eliminated slightly odd identifiers;
|
file |
diff |
annotate
|
Wed, 05 Sep 2012 20:19:37 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Wed, 11 Jan 2012 00:01:54 +0100 |
berghofe |
Removed strange hack introduced in b27e93132603, since equivariance
|
file |
diff |
annotate
|
Sat, 24 Dec 2011 15:53:11 +0100 |
haftmann |
explicitly spelt out proof of equivariance avoids problem with automation due to type constructor `set`
|
file |
diff |
annotate
|
Mon, 12 Sep 2011 07:55:43 +0200 |
nipkow |
new fastforce replacing fastsimp - less confusing name
|
file |
diff |
annotate
|
Mon, 21 Feb 2011 17:43:23 +0100 |
wenzelm |
modernized specifications;
|
file |
diff |
annotate
|
Wed, 08 Sep 2010 19:21:46 +0200 |
haftmann |
modernized primrec
|
file |
diff |
annotate
|
Tue, 02 Mar 2010 09:05:50 +0100 |
haftmann |
repaired subscripts broken in d8d7d1b785af
|
file |
diff |
annotate
|
Mon, 01 Mar 2010 13:40:23 +0100 |
haftmann |
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
|
file |
diff |
annotate
|
Sun, 10 Jan 2010 18:43:45 +0100 |
berghofe |
Adapted to changes in induct method.
|
file |
diff |
annotate
|
Sat, 17 Oct 2009 14:43:18 +0200 |
wenzelm |
eliminated hard tabulators, guessing at each author's individual tab-width;
|
file |
diff |
annotate
|
Wed, 15 Jul 2009 22:30:27 +0200 |
Christian Urban |
simplified proofs
|
file |
diff |
annotate
|
Sun, 26 Apr 2009 00:42:49 +0200 |
Christian Urban |
deleted thm-attributes "fresh" and "bij" (not used); same features can later be implemented by simpler means
|
file |
diff |
annotate
|
Wed, 25 Feb 2009 18:53:34 +0100 |
berghofe |
Added typing and evaluation relations, together with proofs of preservation
|
file |
diff |
annotate
|
Sat, 13 Dec 2008 13:24:45 +0100 |
berghofe |
Modified nominal_primrec to make it work with local theories, unified syntax
|
file |
diff |
annotate
|
Thu, 22 May 2008 16:34:41 +0200 |
urbanc |
made the naming of the induction principles consistent: weak_induct is
|
file |
diff |
annotate
|
Mon, 18 Feb 2008 05:51:16 +0100 |
urbanc |
updated
|
file |
diff |
annotate
|
Wed, 11 Jul 2007 11:36:06 +0200 |
berghofe |
Renamed inductive2 to inductive.
|
file |
diff |
annotate
|
Thu, 14 Jun 2007 23:04:36 +0200 |
wenzelm |
tuned proofs: avoid implicit prems;
|
file |
diff |
annotate
|
Thu, 19 Apr 2007 16:38:59 +0200 |
berghofe |
nominal_inductive no longer proves equivariance.
|
file |
diff |
annotate
|
Wed, 28 Mar 2007 19:16:11 +0200 |
berghofe |
- Renamed <predicate>_eqvt to <predicate>.eqvt
|
file |
diff |
annotate
|
Wed, 28 Mar 2007 18:25:23 +0200 |
urbanc |
the name for the collection of equivariance lemmas is now eqvts (changed from eqvt) in order to avoid clashes with eqvt-lemmas generated in nominal_inductive
|
file |
diff |
annotate
|
Wed, 28 Mar 2007 01:29:43 +0200 |
urbanc |
adapted to nominal_inductive infrastructure
|
file |
diff |
annotate
|
Mon, 12 Mar 2007 11:07:59 +0100 |
berghofe |
Adapted to new inductive definition package.
|
file |
diff |
annotate
|
Tue, 06 Mar 2007 15:28:22 +0100 |
urbanc |
major update of the nominal package; there is now an infrastructure
|
file |
diff |
annotate
|
Mon, 27 Nov 2006 14:00:08 +0100 |
berghofe |
Adapted to new nominal_primrec command.
|
file |
diff |
annotate
|
Wed, 15 Nov 2006 16:23:55 +0100 |
urbanc |
replaced exists_fresh lemma with a version formulated with obtains;
|
file |
diff |
annotate
|
Mon, 23 Oct 2006 00:51:16 +0200 |
berghofe |
Adapted to changes in FCBs.
|
file |
diff |
annotate
|
Mon, 11 Sep 2006 21:35:19 +0200 |
wenzelm |
induct method: renamed 'fixing' to 'arbitrary';
|
file |
diff |
annotate
|
Fri, 18 Aug 2006 18:51:44 +0200 |
urbanc |
adapted using the characteristic equations
|
file |
diff |
annotate
|
Thu, 17 Aug 2006 19:20:43 +0200 |
urbanc |
added definition for size and substitution using the recursion
|
file |
diff |
annotate
|
Sun, 02 Jul 2006 17:27:10 +0200 |
urbanc |
added more infrastructure for the recursion combinator
|
file |
diff |
annotate
|
Fri, 28 Apr 2006 17:59:06 +0200 |
berghofe |
Capitalized theory names.
|
file |
diff |
annotate
|
Sun, 22 Jan 2006 22:16:34 +0100 |
urbanc |
no essential changes
|
file |
diff |
annotate
|
Wed, 11 Jan 2006 18:39:19 +0100 |
urbanc |
cahges to use the new induction-principle (now proved in
|
file |
diff |
annotate
|
Wed, 11 Jan 2006 17:10:11 +0100 |
urbanc |
merged the silly lemmas into the eqvt proof of subtype
|
file |
diff |
annotate
|
Wed, 11 Jan 2006 12:11:53 +0100 |
urbanc |
tuned
|
file |
diff |
annotate
|
Tue, 10 Jan 2006 15:23:31 +0100 |
urbanc |
tuned
|
file |
diff |
annotate
|
Mon, 09 Jan 2006 00:05:10 +0100 |
urbanc |
commented the transitivity and narrowing proof
|
file |
diff |
annotate
|
Wed, 04 Jan 2006 19:53:39 +0100 |
urbanc |
added more documentation; will now try out a modification
|
file |
diff |
annotate
|
Fri, 16 Dec 2005 18:20:03 +0100 |
urbanc |
tuned more proofs
|
file |
diff |
annotate
|
Thu, 15 Dec 2005 21:51:31 +0100 |
urbanc |
there was a small error in the last commit - fixed now
|
file |
diff |
annotate
|
Thu, 15 Dec 2005 21:49:14 +0100 |
urbanc |
tuned more proof and added in-file documentation
|
file |
diff |
annotate
|
Thu, 15 Dec 2005 18:13:40 +0100 |
urbanc |
tuned the proof of transitivity/narrowing
|
file |
diff |
annotate
|
Thu, 15 Dec 2005 11:53:38 +0100 |
urbanc |
made further tunings
|
file |
diff |
annotate
|
Mon, 05 Dec 2005 15:55:19 +0100 |
urbanc |
transitivity should be now in a reasonable state. But
|
file |
diff |
annotate
|
Wed, 30 Nov 2005 19:08:51 +0100 |
urbanc |
started to change the transitivity/narrowing case:
|
file |
diff |
annotate
|