src/Provers/quantifier1.ML
Thu, 30 Oct 2014 16:55:29 +0100 wenzelm eliminated aliases;
Sun, 12 Jan 2014 14:32:22 +0100 wenzelm tuned signature;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Fri, 22 Apr 2011 15:24:00 +0200 wenzelm simplified Data signature;
Fri, 22 Apr 2011 15:05:04 +0200 wenzelm misc tuning and simplification;
Fri, 22 Apr 2011 14:53:11 +0200 wenzelm misc tuning;
Fri, 22 Apr 2011 14:38:49 +0200 wenzelm do not open ML structures;
Fri, 22 Apr 2011 14:30:32 +0200 wenzelm proper context for Quantifier1 simprocs (avoid bad ProofContext.init_global from abc655166d61);
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Tue, 17 Aug 2010 13:10:58 +0200 blanchet merged
Mon, 16 Aug 2010 17:44:27 +0200 blanchet typos in comment
Tue, 17 Aug 2010 12:49:33 +0200 nipkow now works for schematic terms as well, thanks to Alex for the `how-to'
Mon, 03 May 2010 14:25:56 +0200 wenzelm renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
Sat, 13 Mar 2010 16:44:12 +0100 wenzelm removed old CVS Ids;
Mon, 18 May 2009 23:15:38 +0200 nipkow fine-tuned elimination of comprehensions involving x=t.
Sat, 16 May 2009 11:28:02 +0200 nipkow "{x. P x & x=t & Q x}" is now rewritten to "if P t & Q t then {t} else {}"
Sat, 08 Jul 2006 12:54:37 +0200 wenzelm Goal.prove: context;
Fri, 21 Oct 2005 18:14:34 +0200 wenzelm Goal.prove;
Tue, 02 Aug 2005 19:47:12 +0200 wenzelm simprocs: Simplifier.inherit_bounds;
Sun, 13 Feb 2005 17:15:14 +0100 skalberg Deleted Library.option type.
Thu, 08 Jul 2004 19:34:56 +0200 wenzelm adapted type of simprocs;
Thu, 08 Aug 2002 23:46:09 +0200 wenzelm use Tactic.prove instead of prove_goalw_cterm in internal proofs!
Mon, 17 Dec 2001 14:21:59 +0100 nipkow now permutations of quantifiers are allowed as well.
Thu, 29 Mar 2001 13:59:54 +0200 nipkow generalization of 1 point rules for ALL
Fri, 23 Mar 2001 10:12:12 +0100 nipkow added simproc for bounded quantifiers
Wed, 27 Oct 1999 17:17:28 +0200 nipkow Fixed a bug in the EX simproc.
Fri, 28 Nov 1997 07:35:47 +0100 nipkow Quantifier elimination procs.
less more (0) tip