src/HOL/HOL.thy
Sun, 26 Nov 2017 21:08:32 +0100 wenzelm more symbols;
Sun, 22 Oct 2017 09:10:10 +0200 nipkow derived axiom iffI as a lemma (thanks to Alexander Maletzky)
Mon, 09 Oct 2017 19:10:47 +0200 haftmann tuned imports
Sun, 02 Jul 2017 20:13:38 +0200 haftmann proper concept of code declaration wrt. atomicity and Isar declarations
Sat, 17 Jun 2017 15:41:19 +0200 nipkow added simp rules
Sun, 18 Sep 2016 17:59:28 +0200 wenzelm clarified notation: iterated quantifier is negated as one chunk;
Sun, 18 Sep 2016 15:16:42 +0200 wenzelm clarified notation;
Mon, 01 Aug 2016 22:11:29 +0200 wenzelm misc tuning and modernization;
Fri, 29 Jul 2016 09:49:23 +0200 Andreas Lochbihler add lemmas contributed by Peter Gammie
Tue, 12 Apr 2016 14:38:57 +0200 wenzelm Type_Infer.object_logic controls improvement of type inference result;
Fri, 08 Apr 2016 20:15:20 +0200 wenzelm eliminated unused simproc identifier;
Sat, 05 Mar 2016 20:47:31 +0100 wenzelm abbreviations for \<nexists>;
Sat, 05 Mar 2016 19:58:56 +0100 wenzelm old HOL syntax is for input only;
Tue, 23 Feb 2016 16:25:08 +0100 nipkow more canonical names
Tue, 12 Jan 2016 11:49:35 +0100 wenzelm eliminated old defs;
Mon, 28 Dec 2015 21:47:32 +0100 wenzelm former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
Sun, 27 Dec 2015 17:16:21 +0100 wenzelm discontinued ASCII replacement syntax <->;
Tue, 22 Dec 2015 15:39:01 +0100 haftmann stripped some legacy
Mon, 07 Dec 2015 10:38:04 +0100 wenzelm isabelle update_cartouches -c -t;
Fri, 09 Oct 2015 20:26:03 +0200 wenzelm discontinued specific HTML syntax;
Mon, 21 Sep 2015 21:46:14 +0200 wenzelm isabelle update_cartouches;
Mon, 21 Sep 2015 11:31:56 +0200 nipkow Added new simplifier predicate ASSUMPTION
Sun, 13 Sep 2015 22:56:52 +0200 wenzelm tuned proofs -- less legacy;
Wed, 09 Sep 2015 20:57:21 +0200 wenzelm simplified simproc programming interfaces;
Tue, 01 Sep 2015 22:32:58 +0200 wenzelm eliminated \<Colon>;
Sat, 25 Jul 2015 23:41:53 +0200 wenzelm updated to infer_instantiate;
Mon, 20 Jul 2015 11:40:43 +0200 wenzelm proper LaTeX;
Sun, 19 Jul 2015 00:03:10 +0200 wenzelm more symbols;
Sat, 18 Jul 2015 22:58:50 +0200 wenzelm isabelle update_cartouches;
Sat, 09 May 2015 12:19:24 +0200 nipkow undid 6d7b7a037e8d because it does not help but slows simplification down by up to 5% (AODV)
Sun, 03 May 2015 15:38:25 +0200 nipkow swap False to the right in assumptions to be eliminated at the right end
Tue, 28 Apr 2015 19:09:28 +0200 nipkow undid 6d7b7a037e8d
Sat, 25 Apr 2015 17:38:22 +0200 nipkow new ==> simp rule
Wed, 22 Apr 2015 12:11:48 +0200 nipkow added simp rules for ==>
Thu, 09 Apr 2015 20:42:32 +0200 wenzelm clarified keyword 'qualified' in accordance to a similar keyword from Haskell (despite unrelated Binding.qualified in Isabelle/ML);
Wed, 08 Apr 2015 19:39:08 +0200 wenzelm proper context for Object_Logic operations;
Mon, 06 Apr 2015 23:14:05 +0200 wenzelm local setup of induction tools, with restricted access to auxiliary consts;
Mon, 06 Apr 2015 12:37:21 +0200 wenzelm tuned;
Tue, 31 Mar 2015 17:29:44 +0200 nipkow added lemmas
Mon, 23 Mar 2015 15:08:02 +0100 hoelzl fix parameter order of NO_MATCH
Fri, 06 Mar 2015 23:14:41 +0100 wenzelm clarified context;
Fri, 06 Mar 2015 15:58:56 +0100 wenzelm Thm.cterm_of and Thm.ctyp_of operate on local context;
Wed, 04 Mar 2015 22:05:01 +0100 wenzelm clarified signature;
Wed, 04 Mar 2015 19:53:18 +0100 wenzelm tuned signature -- prefer qualified names;
Wed, 11 Feb 2015 12:01:56 +0000 paulson Merge
Tue, 10 Feb 2015 16:08:11 +0000 paulson New lemmas and a bit of tidying up.
Tue, 10 Feb 2015 16:46:21 +0100 wenzelm misc tuning;
Tue, 10 Feb 2015 14:48:26 +0100 wenzelm proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
Sat, 22 Nov 2014 11:36:00 +0100 wenzelm named_theorems: multiple args;
Mon, 10 Nov 2014 21:49:48 +0100 wenzelm proper context for assume_tac (atac remains as fall-back without context);
Sun, 09 Nov 2014 18:27:43 +0100 wenzelm proper context;
Sun, 09 Nov 2014 17:04:14 +0100 wenzelm proper context for match_tac etc.;
Sun, 09 Nov 2014 14:08:00 +0100 wenzelm proper context for compose_tac, Splitter.split_tac (relevant for unify trace options);
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Thu, 30 Oct 2014 22:45:19 +0100 wenzelm eliminated aliases;
Thu, 30 Oct 2014 09:15:54 +0100 hoelzl disable coercions for NO_MATCH
Wed, 29 Oct 2014 19:01:49 +0100 wenzelm modernized setup;
Fri, 24 Oct 2014 15:07:49 +0200 hoelzl move NO_MATCH simproc from the AFP entry Graph_Theory to HOL
Mon, 13 Oct 2014 18:45:48 +0200 wenzelm Local_Interpretation is superseded by Plugin with formal Plugin_Name management, avoiding undeclared strings;
Sat, 16 Aug 2014 22:14:57 +0200 wenzelm updated to named_theorems;
less more (0) -300 -100 -60 tip