wenzelm [Sat, 15 Sep 2007 19:25:54 +0200] rev 24580
replaced Symbol.is_hex_letter to Symbol.is_ascii_hex;
tuned Symbol.is_ascii_blank (according to SML syntax);
wenzelm [Sat, 15 Sep 2007 19:25:43 +0200] rev 24579
Lexical syntax for SML.
wenzelm [Sat, 15 Sep 2007 19:25:32 +0200] rev 24578
added ML/ml_lex.ML;
wenzelm [Sat, 15 Sep 2007 19:25:19 +0200] rev 24577
removed redundant OuterLex.make_lexicon;
krauss [Fri, 14 Sep 2007 22:22:53 +0200] rev 24576
lexicographic_order method uses "<*mlex*>" instead of "measures" => no longer depends on List.thy
krauss [Fri, 14 Sep 2007 22:21:46 +0200] rev 24575
added "<*mlex*>" which lexicographically combines a measure function with a relation
wenzelm [Fri, 14 Sep 2007 17:02:34 +0200] rev 24574
moved ML_XXX.ML files to Pure/ML;
paulson [Fri, 14 Sep 2007 15:27:12 +0200] rev 24573
tidied
urbanc [Fri, 14 Sep 2007 13:32:07 +0200] rev 24572
reverted back to the old version of the equivariance lemma for ALL
urbanc [Thu, 13 Sep 2007 23:58:38 +0200] rev 24571
some cleaning up to do with contexts
berghofe [Thu, 13 Sep 2007 18:11:59 +0200] rev 24570
Generalized equivariance and nominal_inductive commands to
inductive definitions involving arbitrary monotone operators.
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.