Fri, 15 Nov 2024 23:20:24 +0100 |
wenzelm |
tuned proofs;
|
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
|
Tue, 14 Mar 2023 18:19:10 +0100 |
nipkow |
Adjusted to new map update priorities
|
file |
diff |
annotate
|
Sat, 05 Jan 2019 17:24:33 +0100 |
wenzelm |
isabelle update -u control_cartouches;
|
file |
diff |
annotate
|
Fri, 15 Jun 2018 13:02:12 +0200 |
nipkow |
empty -> Map.empty
|
file |
diff |
annotate
|
Thu, 15 Feb 2018 12:11:00 +0100 |
wenzelm |
more symbols;
|
file |
diff |
annotate
|
Tue, 23 Feb 2016 16:25:08 +0100 |
nipkow |
more canonical names
|
file |
diff |
annotate
|
Sat, 02 Jan 2016 18:48:45 +0100 |
wenzelm |
isabelle update_cartouches -c -t;
|
file |
diff |
annotate
|
Wed, 01 Apr 2015 18:18:12 +0200 |
wenzelm |
evade popular keyword;
|
file |
diff |
annotate
|
Sun, 02 Nov 2014 18:16:19 +0100 |
wenzelm |
modernized header;
|
file |
diff |
annotate
|
Sun, 16 Feb 2014 18:39:40 +0100 |
blanchet |
folded 'Option.set' into BNF-generated 'set_option'
|
file |
diff |
annotate
|
Thu, 16 May 2013 17:39:38 +0200 |
wenzelm |
tuned signature -- depend on context by default;
|
file |
diff |
annotate
|
Thu, 18 Apr 2013 17:07:01 +0200 |
wenzelm |
simplifier uses proper Proof.context instead of historic type simpset;
|
file |
diff |
annotate
|
Fri, 12 Apr 2013 17:21:51 +0200 |
wenzelm |
modifiers for classical wrappers operate on Proof.context instead of claset;
|
file |
diff |
annotate
|
Wed, 28 Mar 2012 12:08:08 +0200 |
wenzelm |
simplified statements and proofs;
|
file |
diff |
annotate
|
Sat, 14 Jan 2012 16:14:22 +0100 |
wenzelm |
tuned white space;
|
file |
diff |
annotate
|
Sun, 20 Nov 2011 21:28:07 +0100 |
wenzelm |
eliminated obsolete "standard";
|
file |
diff |
annotate
|
Sun, 20 Nov 2011 21:05:23 +0100 |
wenzelm |
eliminated obsolete "standard";
|
file |
diff |
annotate
|
Mon, 12 Sep 2011 07:55:43 +0200 |
nipkow |
new fastforce replacing fastsimp - less confusing name
|
file |
diff |
annotate
|
Mon, 26 Jul 2010 17:41:26 +0200 |
wenzelm |
modernized/unified some specifications;
|
file |
diff |
annotate
|
Thu, 01 Jul 2010 16:54:44 +0200 |
haftmann |
"prod" and "sum" replace "*" and "+" respectively
|
file |
diff |
annotate
|
Tue, 02 Mar 2010 12:26:50 +0100 |
krauss |
killed more recdefs
|
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
|
Wed, 10 Feb 2010 00:45:16 +0100 |
wenzelm |
modernized syntax translations, using mostly abbreviation/notation;
|
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, 04 Mar 2009 10:47:20 +0100 |
nipkow |
Made Option a separate theory and renamed option_map to Option.map
|
file |
diff |
annotate
|
Tue, 07 Oct 2008 16:07:50 +0200 |
haftmann |
arbitrary is undefined
|
file |
diff |
annotate
|
Sat, 28 Jul 2007 20:40:22 +0200 |
wenzelm |
tuned ML/simproc declarations;
|
file |
diff |
annotate
|
Wed, 13 Jun 2007 00:01:41 +0200 |
wenzelm |
tuned proofs: avoid implicit prems;
|
file |
diff |
annotate
|
Fri, 09 Mar 2007 08:45:55 +0100 |
haftmann |
*** empty log message ***
|
file |
diff |
annotate
|
Mon, 11 Dec 2006 16:06:14 +0100 |
berghofe |
Adapted to new inductive definition package.
|
file |
diff |
annotate
|
Mon, 17 Oct 2005 23:10:13 +0200 |
wenzelm |
change_claset/simpset;
|
file |
diff |
annotate
|
Fri, 17 Jun 2005 16:12:49 +0200 |
haftmann |
migrated theory headers to new format
|
file |
diff |
annotate
|
Mon, 21 Jun 2004 10:25:57 +0200 |
kleing |
Merged in license change from Isabelle2004
|
file |
diff |
annotate
|
Fri, 29 Aug 2003 15:19:02 +0200 |
ballarin |
Methods rule_tac etc support static (Isar) contexts.
|
file |
diff |
annotate
|
Wed, 14 May 2003 20:29:18 +0200 |
schirmer |
Adapted to changes in Map.thy
|
file |
diff |
annotate
|
Wed, 14 May 2003 10:22:09 +0200 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Thu, 31 Oct 2002 18:27:10 +0100 |
schirmer |
"Definite Assignment Analysis" included, with proof of correctness. Large adjustments of type safety proof and soundness proof of the axiomatic semantics were necessary. Completeness proof of the loop rule of the axiomatic semantic was altered. So the additional polymorphic variants of some rules could be removed.
|
file |
diff |
annotate
|
Mon, 30 Sep 2002 16:14:02 +0200 |
berghofe |
Adapted to new simplifier.
|
file |
diff |
annotate
|
Wed, 27 Feb 2002 15:23:42 +0100 |
schirmer |
Some simple properties of dynamic accessibility added.
|
file |
diff |
annotate
|
Wed, 27 Feb 2002 08:52:09 +0100 |
schirmer |
Cleaning up the definition of static overriding.
|
file |
diff |
annotate
|
Mon, 25 Feb 2002 20:48:14 +0100 |
wenzelm |
clarified syntax of ``long'' statements: fixes/assumes/shows;
|
file |
diff |
annotate
|
Fri, 22 Feb 2002 11:26:44 +0100 |
schirmer |
Added check for field/method access to operational semantics and proved the acesses valid.
|
file |
diff |
annotate
|
Fri, 15 Feb 2002 20:41:39 +0100 |
wenzelm |
replaced nodups by distinct;
|
file |
diff |
annotate
|
Mon, 28 Jan 2002 18:51:48 +0100 |
wenzelm |
GPLed;
|
file |
diff |
annotate
|
Mon, 28 Jan 2002 18:50:23 +0100 |
wenzelm |
tuned header;
|
file |
diff |
annotate
|
Mon, 28 Jan 2002 17:00:19 +0100 |
schirmer |
Isabelle/Bali sources;
|
file |
diff |
annotate
|