Sat, 03 Nov 2001 01:36:19 +0100 |
wenzelm |
moved into Main;
|
changeset |
files
|
Sat, 03 Nov 2001 01:35:11 +0100 |
wenzelm |
moved String into Main;
|
changeset |
files
|
Sat, 03 Nov 2001 01:33:54 +0100 |
wenzelm |
tuned;
|
changeset |
files
|
Sat, 03 Nov 2001 01:33:33 +0100 |
wenzelm |
HOLCF: proper rep_datatype lift (see theory Lift); use plain induct_tac
|
changeset |
files
|
Fri, 02 Nov 2001 22:02:41 +0100 |
wenzelm |
declare transitive;
|
changeset |
files
|
Fri, 02 Nov 2001 22:01:58 +0100 |
wenzelm |
theory Calculation move to Set;
|
changeset |
files
|
Fri, 02 Nov 2001 22:01:07 +0100 |
wenzelm |
transitive declared in Pure;
|
changeset |
files
|
Fri, 02 Nov 2001 17:55:24 +0100 |
paulson |
Numerals and simprocs for types real and hypreal. The abstract
|
changeset |
files
|
Thu, 01 Nov 2001 21:12:13 +0100 |
wenzelm |
Goals.add_locale;
|
changeset |
files
|
Thu, 01 Nov 2001 21:11:52 +0100 |
wenzelm |
fix_frees;
|
changeset |
files
|
Thu, 01 Nov 2001 21:11:17 +0100 |
wenzelm |
theorem: locale argument;
|
changeset |
files
|
Thu, 01 Nov 2001 21:10:47 +0100 |
wenzelm |
beginnings of new locales (not yet functional);
|
changeset |
files
|
Thu, 01 Nov 2001 21:10:13 +0100 |
wenzelm |
Goals.setup;
|
changeset |
files
|
Thu, 01 Nov 2001 21:09:53 +0100 |
wenzelm |
parking code for old-style locales here;
|
changeset |
files
|
Wed, 31 Oct 2001 22:05:37 +0100 |
wenzelm |
tuned notation (degree instead of dollar);
|
changeset |
files
|
Wed, 31 Oct 2001 22:04:29 +0100 |
wenzelm |
theorem(_i): locale argument;
|
changeset |
files
|
Wed, 31 Oct 2001 22:02:33 +0100 |
wenzelm |
Proof.init_state thy None;
|
changeset |
files
|
Wed, 31 Oct 2001 22:02:11 +0100 |
wenzelm |
simplified export;
|
changeset |
files
|
Wed, 31 Oct 2001 22:00:25 +0100 |
wenzelm |
'atomize': CHANGED_PROP;
|
changeset |
files
|
Wed, 31 Oct 2001 22:00:02 +0100 |
wenzelm |
global statements: locale argument;
|
changeset |
files
|
Wed, 31 Oct 2001 21:59:25 +0100 |
wenzelm |
added local_standard;
|
changeset |
files
|
Wed, 31 Oct 2001 21:59:07 +0100 |
wenzelm |
IsarThy.theorem_i: no locale;
|
changeset |
files
|
Wed, 31 Oct 2001 21:58:04 +0100 |
wenzelm |
removed obsolete (rule equal_intr_rule);
|
changeset |
files
|
Wed, 31 Oct 2001 20:00:35 +0100 |
berghofe |
Additional rules for simplifying inside "Goal"
|
changeset |
files
|
Wed, 31 Oct 2001 19:59:21 +0100 |
berghofe |
- Tuned add_cnstrt
|
changeset |
files
|
Wed, 31 Oct 2001 19:49:36 +0100 |
berghofe |
Removed name_thm from finish_global.
|
changeset |
files
|
Wed, 31 Oct 2001 19:41:29 +0100 |
berghofe |
Tuned function thm_proof.
|
changeset |
files
|
Wed, 31 Oct 2001 19:37:04 +0100 |
berghofe |
- enter_thmx -> enter_thms
|
changeset |
files
|
Wed, 31 Oct 2001 19:32:05 +0100 |
berghofe |
norm_hhf_eq is now stored using open_store_standard_thm.
|
changeset |
files
|
Wed, 31 Oct 2001 01:28:39 +0100 |
wenzelm |
induct: internalize ``missing'' consumes-facts from goal state
|
changeset |
files
|
Wed, 31 Oct 2001 01:27:04 +0100 |
wenzelm |
- 'induct' may now use elim-style induction rules without chaining
|
changeset |
files
|
Wed, 31 Oct 2001 01:26:42 +0100 |
wenzelm |
(induct set: ...);
|
changeset |
files
|
Wed, 31 Oct 2001 01:22:27 +0100 |
wenzelm |
put_consumes: really overwrite existing tag;
|
changeset |
files
|
Wed, 31 Oct 2001 01:21:56 +0100 |
wenzelm |
finish_global: Tactic.norm_hhf;
|
changeset |
files
|
Wed, 31 Oct 2001 01:21:31 +0100 |
wenzelm |
use HOL.induct_XXX;
|
changeset |
files
|
Wed, 31 Oct 2001 01:21:01 +0100 |
wenzelm |
use induct_rulify2;
|
changeset |
files
|
Wed, 31 Oct 2001 01:20:42 +0100 |
wenzelm |
renamed inductive_XXX to induct_XXX;
|
changeset |
files
|
Wed, 31 Oct 2001 01:19:58 +0100 |
wenzelm |
induct_impliesI;
|
changeset |
files
|
Tue, 30 Oct 2001 17:37:25 +0100 |
wenzelm |
tuned induct proofs;
|
changeset |
files
|
Tue, 30 Oct 2001 17:33:56 +0100 |
wenzelm |
- 'induct' method now derives symbolic cases from the *rulified* rule
|
changeset |
files
|
Tue, 30 Oct 2001 17:33:03 +0100 |
wenzelm |
tuned;
|
changeset |
files
|
Tue, 30 Oct 2001 17:30:21 +0100 |
wenzelm |
induct: cases are extracted from rulified rule;
|
changeset |
files
|
Tue, 30 Oct 2001 17:29:43 +0100 |
wenzelm |
removed obsolete make_raw;
|
changeset |
files
|
Tue, 30 Oct 2001 13:43:26 +0100 |
wenzelm |
lemma Least_mono moved from Typedef.thy to Set.thy;
|
changeset |
files
|
Mon, 29 Oct 2001 17:22:18 +0100 |
wenzelm |
tuned;
|
changeset |
files
|
Mon, 29 Oct 2001 14:09:10 +0100 |
wenzelm |
removed option -depend (not available everywhere?);
|
changeset |
files
|
Sun, 28 Oct 2001 22:59:12 +0100 |
wenzelm |
converted theory "Set";
|
changeset |
files
|
Sun, 28 Oct 2001 22:58:39 +0100 |
wenzelm |
fixed string_of_mixfix;
|
changeset |
files
|
Sun, 28 Oct 2001 21:14:56 +0100 |
wenzelm |
tuned declaration of rules;
|
changeset |
files
|
Sun, 28 Oct 2001 21:10:47 +0100 |
wenzelm |
equal_intr_rule already declared in Pure;
|
changeset |
files
|
Sun, 28 Oct 2001 19:44:58 +0100 |
wenzelm |
rules for meta-level conjunction;
|
changeset |
files
|
Sun, 28 Oct 2001 19:44:26 +0100 |
wenzelm |
tuned prove;
|
changeset |
files
|
Sat, 27 Oct 2001 23:21:19 +0200 |
wenzelm |
tuned;
|
changeset |
files
|
Sat, 27 Oct 2001 23:19:55 +0200 |
wenzelm |
added prove;
|
changeset |
files
|
Sat, 27 Oct 2001 23:19:37 +0200 |
wenzelm |
declare equal_intr_rule as intro;
|
changeset |
files
|
Sat, 27 Oct 2001 23:19:04 +0200 |
wenzelm |
tuned prove;
|
changeset |
files
|
Sat, 27 Oct 2001 23:18:40 +0200 |
wenzelm |
removed obsolete goal_subclass, goal_arity;
|
changeset |
files
|
Sat, 27 Oct 2001 23:17:46 +0200 |
wenzelm |
use Tactic.prove;
|
changeset |
files
|
Sat, 27 Oct 2001 23:17:28 +0200 |
wenzelm |
use Tactic.prove;
|
changeset |
files
|
Sat, 27 Oct 2001 23:16:15 +0200 |
wenzelm |
tuned;
|
changeset |
files
|