| Sat, 27 Apr 2013 20:50:20 +0200 |
wenzelm |
uniform Proof.context for hyp_subst_tac;
|
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, 28 Feb 2013 17:14:55 +0100 |
wenzelm |
provide common HOLogic.conj_conv and HOLogic.eq_conv;
|
file |
diff |
annotate
|
| Thu, 28 Feb 2013 16:54:52 +0100 |
wenzelm |
just one HOLogic.Trueprop_conv, with regular exception CTERM;
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 19:55:37 +0100 |
bulwahn |
using hyp_subst_tac that allows to pass the current simpset to avoid the renamed bound variable warning in the simplifier
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 19:55:17 +0100 |
bulwahn |
rewriting with the simpset that is passed to the simproc
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 17:11:04 +0100 |
bulwahn |
handling x : S y pattern with the default mechanism instead of raising an exception in the set_comprehension_pointfree simproc
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 17:06:59 +0100 |
bulwahn |
tuned
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 16:25:26 +0100 |
bulwahn |
syntactic tuning and restructuring of set_comprehension_pointfree simproc
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 11:59:50 +0100 |
bulwahn |
using more proper simpset in tactic of set_comprehension_pointfree simproc to avoid renamed bound variable warnings in recursive simplifier calls
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 11:59:49 +0100 |
bulwahn |
improving the extension of sets in case of more than one bound variable; rearranging the tactic to prefer simpler steps before more involved ones
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 11:59:47 +0100 |
bulwahn |
importing term with schematic type variables properly before passing it to the tactic in the set_comprehension_pointfree simproc
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 11:59:47 +0100 |
bulwahn |
handling arbitrary terms in the set comprehension and more general merging of patterns possible in the set_comprehension_pointfree simproc
|
file |
diff |
annotate
|
| Thu, 08 Nov 2012 11:59:46 +0100 |
bulwahn |
simplified structure of patterns in set_comprehension_simproc
|
file |
diff |
annotate
|
| Sun, 21 Oct 2012 08:39:41 +0200 |
bulwahn |
another refinement in the comprehension conversion
|
file |
diff |
annotate
|
| Sun, 21 Oct 2012 05:24:59 +0200 |
bulwahn |
refined simplifier call in comprehension_conv
|
file |
diff |
annotate
|
| Sun, 21 Oct 2012 05:24:56 +0200 |
bulwahn |
passing around the simpset instead of the context; rewriting tactics to avoid the 'renamed bound variable' warnings in nested simplifier calls
|
file |
diff |
annotate
|
| Sat, 20 Oct 2012 09:09:35 +0200 |
bulwahn |
improving tactic in setcomprehension_simproc
|
file |
diff |
annotate
|
| Sat, 20 Oct 2012 09:09:33 +0200 |
bulwahn |
tuned tactic in set_comprehension_pointfree simproc to handle composition of negation and vimage
|
file |
diff |
annotate
|
| Sat, 20 Oct 2012 09:09:32 +0200 |
bulwahn |
passing names and types of all bounds around in the simproc
|
file |
diff |
annotate
|
| Thu, 18 Oct 2012 10:06:27 +0200 |
bulwahn |
locally inverting previously applied simplifications with ex_simps in set_comprehension_pointfree
|
file |
diff |
annotate
|
| Wed, 17 Oct 2012 15:25:52 +0200 |
bulwahn |
comprehension conversion reuses suggested names for bound variables instead of invented fresh ones; tuned tactic
|
file |
diff |
annotate
|
| Wed, 17 Oct 2012 14:13:57 +0200 |
bulwahn |
checking for bound variables in the set expression; handling negation more generally
|
file |
diff |
annotate
|
| Wed, 17 Oct 2012 14:13:57 +0200 |
bulwahn |
refined conversion to only react on proper set comprehensions; tuned
|
file |
diff |
annotate
|
| Wed, 17 Oct 2012 14:13:57 +0200 |
bulwahn |
employing a preprocessing conversion that rewrites {(x1, ..., xn). P x1 ... xn} to {(x1, ..., xn) | x1 ... xn. P x1 ... xn} in set_comprehension_pointfree simproc
|
file |
diff |
annotate
|
| Tue, 16 Oct 2012 13:18:13 +0200 |
bulwahn |
tactic of set_comprehension_pointfree simproc handles f x y : S patterns with Set.vimage
|
file |
diff |
annotate
|
| Tue, 16 Oct 2012 13:18:12 +0200 |
bulwahn |
term construction of set_comprehension_pointfree simproc handles f x y : S patterns with Set.vimage
|
file |
diff |
annotate
|
| Tue, 16 Oct 2012 13:18:10 +0200 |
bulwahn |
extending preprocessing of simproc to rewrite subset inequality into membership of powerset
|
file |
diff |
annotate
|
| Mon, 15 Oct 2012 16:18:48 +0200 |
bulwahn |
setcomprehension_pointfree simproc also works for set comprehension without an equation
|
file |
diff |
annotate
|
| Sun, 14 Oct 2012 19:16:35 +0200 |
bulwahn |
refined tactic in set_comprehension_pointfree simproc
|
file |
diff |
annotate
|