berghofe [Thu, 13 Sep 2007 18:08:08 +0200] rev 24569
Added equivariance lemmas for induct_forall.
berghofe [Thu, 13 Sep 2007 18:06:50 +0200] rev 24568
Added equivariance lemma for induct_implies.
webertj [Tue, 11 Sep 2007 14:26:49 +0200] rev 24567
typo fixed, dead link removed
nipkow [Mon, 10 Sep 2007 19:21:03 +0200] rev 24566
added lemma
berghofe [Mon, 10 Sep 2007 16:09:01 +0200] rev 24565
Auto quickcheck now displays counterexample using Proof.goal_message
rather than producing an error message.
wenzelm [Sat, 08 Sep 2007 20:37:22 +0200] rev 24564
added String.isSubstring;
wenzelm [Sat, 08 Sep 2007 19:58:39 +0200] rev 24563
export is_finished;
added thy_ord (based on update_time);
begin_thy/register_thy: more precise handling of update_time;
wenzelm [Sat, 08 Sep 2007 19:58:38 +0200] rev 24562
Present.session_name;
wenzelm [Sat, 08 Sep 2007 19:58:37 +0200] rev 24561
tuned signature;
tuned message;
wenzelm [Sat, 08 Sep 2007 19:58:36 +0200] rev 24560
thy_deps: ThyInfo.thy_ord, improved dir/unfold entry;
wenzelm [Sat, 08 Sep 2007 19:58:35 +0200] rev 24559
removed thy_ord (erratic due to multi-threading);
urbanc [Sat, 08 Sep 2007 18:30:02 +0200] rev 24558
some cleaning up
wenzelm [Fri, 07 Sep 2007 22:13:49 +0200] rev 24557
theorem: apply hook last;
wenzelm [Fri, 07 Sep 2007 22:13:48 +0200] rev 24556
reset goal messages after goal update;
wenzelm [Fri, 07 Sep 2007 22:13:45 +0200] rev 24555
added hilite markup;
wenzelm [Fri, 07 Sep 2007 20:40:08 +0200] rev 24554
fixed type alias in signature;
nipkow [Fri, 07 Sep 2007 17:56:03 +0200] rev 24553
added lemma
paulson [Fri, 07 Sep 2007 15:35:25 +0200] rev 24552
allow TVars during type inference
paulson [Fri, 07 Sep 2007 15:34:32 +0200] rev 24551
tidied the proofs
wenzelm [Fri, 07 Sep 2007 09:11:32 +0200] rev 24550
made smlnj happy;
paulson [Thu, 06 Sep 2007 18:19:00 +0200] rev 24549
new fun declaration
paulson [Thu, 06 Sep 2007 17:06:04 +0200] rev 24548
Auto-config of E_HOME, SPASS_HOME, VAMPIRE_HOME
paulson [Thu, 06 Sep 2007 17:03:53 +0200] rev 24547
Vampire structured proofs. Better parsing; some bug fixes.
paulson [Thu, 06 Sep 2007 17:03:32 +0200] rev 24546
chained facts are now included
paulson [Thu, 06 Sep 2007 16:54:03 +0200] rev 24545
new proofs found
urbanc [Thu, 06 Sep 2007 16:28:42 +0200] rev 24544
trivial cleaning up
wenzelm [Thu, 06 Sep 2007 12:30:41 +0200] rev 24543
added goal_message;
wenzelm [Thu, 06 Sep 2007 12:30:11 +0200] rev 24542
theorem hooks: apply in declaration order;
berghofe [Thu, 06 Sep 2007 11:53:17 +0200] rev 24541
Generalized code generator for numerals.
berghofe [Thu, 06 Sep 2007 11:52:13 +0200] rev 24540
- New theories Lambda/NormalForm and Lambda/Standardization
- Integrated Executable_Rat and Executable_Real theories into
Rational and RealDef theories