Thu, 06 Mar 2014 10:11:38 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Sat, 14 Dec 2013 17:28:05 +0100 |
wenzelm |
proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
|
file |
diff |
annotate
|
Fri, 23 Aug 2013 17:01:12 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Sat, 27 Jul 2013 16:35:51 +0200 |
wenzelm |
standardized aliases;
|
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
|
Thu, 03 Nov 2011 22:51:37 +0100 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Wed, 12 Oct 2011 22:21:38 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Wed, 27 Apr 2011 17:58:45 +0200 |
wenzelm |
reorganized fixes as specialized (global) name space;
|
file |
diff |
annotate
|
Sat, 16 Apr 2011 16:15:37 +0200 |
wenzelm |
modernized structure Proof_Context;
|
file |
diff |
annotate
|
Wed, 26 May 2010 16:17:30 +0200 |
haftmann |
dropped legacy theorem bindings
|
file |
diff |
annotate
|
Mon, 17 May 2010 23:54:15 +0200 |
wenzelm |
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
|
file |
diff |
annotate
|
Sun, 10 Jan 2010 18:01:04 +0100 |
berghofe |
Added infrastructure for simplifying equality constraints.
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 09:13:46 +0100 |
haftmann |
normalized uncurry take/drop
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 17:28:25 +0100 |
haftmann |
curried take/drop
|
file |
diff |
annotate
|
Sun, 01 Nov 2009 15:24:45 +0100 |
wenzelm |
modernized structure Rule_Cases;
|
file |
diff |
annotate
|
Thu, 15 Oct 2009 23:28:10 +0200 |
wenzelm |
replaced String.concat by implode;
|
file |
diff |
annotate
|
Mon, 16 Mar 2009 18:24:30 +0100 |
wenzelm |
simplified method setup;
|
file |
diff |
annotate
|
Fri, 13 Mar 2009 19:58:26 +0100 |
wenzelm |
unified type Proof.method and pervasive METHOD combinators;
|
file |
diff |
annotate
|
Wed, 25 Feb 2009 19:34:00 +0100 |
berghofe |
Added lemmas for normalizing freshness results involving fresh_star.
|
file |
diff |
annotate
|
Wed, 21 Jan 2009 16:47:32 +0100 |
haftmann |
binding is alias for Binding.T
|
file |
diff |
annotate
|
Thu, 04 Dec 2008 14:43:33 +0100 |
haftmann |
cleaned up binding module and related code
|
file |
diff |
annotate
|
Tue, 02 Sep 2008 14:10:45 +0200 |
wenzelm |
explicit type Name.binding for higher-specification elements;
|
file |
diff |
annotate
|
Sat, 09 Aug 2008 22:43:46 +0200 |
wenzelm |
unified Args.T with OuterLex.token, renamed some operations;
|
file |
diff |
annotate
|
Thu, 26 Jun 2008 15:06:25 +0200 |
wenzelm |
Args.context;
|
file |
diff |
annotate
|
Sun, 18 May 2008 15:04:17 +0200 |
wenzelm |
guess_instance: proper context;
|
file |
diff |
annotate
|
Thu, 17 Apr 2008 22:22:23 +0200 |
wenzelm |
adapted to ProofContext.revert_skolem: extra Name.clean required;
|
file |
diff |
annotate
|
Sat, 26 Jan 2008 20:01:37 +0100 |
wenzelm |
avoid redundant escaping of Isabelle symbols;
|
file |
diff |
annotate
|
Tue, 09 Oct 2007 00:20:13 +0200 |
wenzelm |
generic Syntax.pretty/string_of operations;
|
file |
diff |
annotate
|
Thu, 04 Oct 2007 14:42:47 +0200 |
wenzelm |
moved Pure/Isar/induct_attrib.ML and Provers/induct_method.ML to Tools/induct.ML;
|
file |
diff |
annotate
|
Thu, 05 Jul 2007 20:01:28 +0200 |
wenzelm |
simplified ObjectLogic.atomize;
|
file |
diff |
annotate
|
Tue, 16 Jan 2007 10:25:38 +0100 |
urbanc |
added capabilities to handle mutual inductions
|
file |
diff |
annotate
|
Mon, 18 Dec 2006 08:21:35 +0100 |
haftmann |
switched argument order in *.syntax lifters
|
file |
diff |
annotate
|
Thu, 12 Oct 2006 22:03:33 +0200 |
urbanc |
To be consistent with "induct", I renamed "fixing" to "arbitrary".
|
file |
diff |
annotate
|
Wed, 02 Aug 2006 22:26:40 +0200 |
wenzelm |
simplified Assumption/ProofContext.export;
|
file |
diff |
annotate
|
Tue, 11 Jul 2006 12:16:57 +0200 |
wenzelm |
Name.internal;
|
file |
diff |
annotate
|
Sat, 17 Jun 2006 19:37:43 +0200 |
wenzelm |
RuleCases.mutual_rule: ctxt;
|
file |
diff |
annotate
|
Tue, 21 Feb 2006 15:06:50 +0100 |
wenzelm |
distinct (op =);
|
file |
diff |
annotate
|
Mon, 13 Feb 2006 17:02:54 +0100 |
berghofe |
Adapted to Context.generic syntax.
|
file |
diff |
annotate
|
Sat, 07 Jan 2006 12:28:25 +0100 |
wenzelm |
RuleCases.make_nested;
|
file |
diff |
annotate
|
Thu, 05 Jan 2006 17:16:40 +0100 |
wenzelm |
proper handling of simultaneous goals and mutual rules;
|
file |
diff |
annotate
|
Thu, 01 Dec 2005 04:46:17 +0100 |
urbanc |
changed "fresh:" to "avoiding:" and cleaned up the weakening example
|
file |
diff |
annotate
|
Wed, 30 Nov 2005 15:24:32 +0100 |
wenzelm |
added rename_params_rule: recover orginal fresh names in subgoals/cases;
|
file |
diff |
annotate
|
Wed, 30 Nov 2005 14:27:50 +0100 |
wenzelm |
fresh: frees instead of terms, rename corresponding params in rule;
|
file |
diff |
annotate
|
Wed, 30 Nov 2005 00:46:08 +0100 |
wenzelm |
proper treatment of tuple/tuple_fun -- nest to the left!
|
file |
diff |
annotate
|
Tue, 29 Nov 2005 18:09:12 +0100 |
wenzelm |
reworked version with proper support for defs, fixes, fresh specification;
|
file |
diff |
annotate
|
Sun, 27 Nov 2005 05:09:43 +0100 |
urbanc |
some minor tunings
|
file |
diff |
annotate
|
Sun, 13 Nov 2005 22:36:30 +0100 |
urbanc |
changed the HOL_basic_ss back and selectively added
|
file |
diff |
annotate
|
Sun, 13 Nov 2005 20:33:36 +0100 |
urbanc |
exchanged HOL_ss for HOL_basic_ss in the simplification
|
file |
diff |
annotate
|
Mon, 07 Nov 2005 10:47:25 +0100 |
urbanc |
fixed bug with nominal induct
|
file |
diff |
annotate
|
Tue, 01 Nov 2005 23:54:29 +0100 |
urbanc |
tunings of some comments (nothing serious)
|
file |
diff |
annotate
|
Mon, 17 Oct 2005 12:30:57 +0200 |
berghofe |
Initial revision.
|
file |
diff |
annotate
|