paulson [Mon, 05 Nov 2001 13:55:48 +0100] rev 12051
new Sqrt example
wenzelm [Sun, 04 Nov 2001 21:12:03 +0100] rev 12050
tuned comment;
wenzelm [Sun, 04 Nov 2001 21:00:28 +0100] rev 12049
simplified Proof.init_state:
wenzelm [Sun, 04 Nov 2001 21:00:06 +0100] rev 12048
added get_thms_with_closure;
fix_frees: only new ones;
wenzelm [Sun, 04 Nov 2001 20:59:01 +0100] rev 12047
added locale_element;
wenzelm [Sun, 04 Nov 2001 20:58:26 +0100] rev 12046
locale elements;
wenzelm [Sun, 04 Nov 2001 20:58:01 +0100] rev 12045
theorem(_i): locale elements;
wenzelm [Sun, 04 Nov 2001 20:57:29 +0100] rev 12044
locale syntax;
wenzelm [Sun, 04 Nov 2001 20:56:59 +0100] rev 12043
IsarThy.theorem_i (None, []);
wenzelm [Sun, 04 Nov 2001 20:56:19 +0100] rev 12042
updated;
berghofe [Sat, 03 Nov 2001 18:49:40 +0100] rev 12041
Fixed bug in function add_npvars.
wenzelm [Sat, 03 Nov 2001 18:44:49 +0100] rev 12040
updated;
wenzelm [Sat, 03 Nov 2001 18:42:55 +0100] rev 12039
tuned;
wenzelm [Sat, 03 Nov 2001 18:42:38 +0100] rev 12038
proper use of bind_thm(s);
wenzelm [Sat, 03 Nov 2001 18:42:00 +0100] rev 12037
adapted to new-style theories;
wenzelm [Sat, 03 Nov 2001 18:41:28 +0100] rev 12036
GPLed;
wenzelm [Sat, 03 Nov 2001 18:41:13 +0100] rev 12035
converted theory Dnat;
wenzelm [Sat, 03 Nov 2001 18:40:21 +0100] rev 12034
* 'domain' package adapted to new-style theories, e.g. see
HOLCF/ex/Dnat.thy;
wenzelm [Sat, 03 Nov 2001 01:45:32 +0100] rev 12033
document setup;
wenzelm [Sat, 03 Nov 2001 01:44:45 +0100] rev 12032
replaced Undef by UU;
wenzelm [Sat, 03 Nov 2001 01:44:26 +0100] rev 12031
ax_flat;
wenzelm [Sat, 03 Nov 2001 01:41:26 +0100] rev 12030
GPLed;
wenzelm [Sat, 03 Nov 2001 01:40:28 +0100] rev 12029
tuned;
wenzelm [Sat, 03 Nov 2001 01:39:17 +0100] rev 12028
replaced Undef by UU;
wenzelm [Sat, 03 Nov 2001 01:38:39 +0100] rev 12027
converted theory Lift;
wenzelm [Sat, 03 Nov 2001 01:38:11 +0100] rev 12026
rep_datatype lift;
converted to new-style theory;
wenzelm [Sat, 03 Nov 2001 01:36:19 +0100] rev 12025
moved into Main;
wenzelm [Sat, 03 Nov 2001 01:35:11 +0100] rev 12024
moved String into Main;
wenzelm [Sat, 03 Nov 2001 01:33:54 +0100] rev 12023
tuned;
wenzelm [Sat, 03 Nov 2001 01:33:33 +0100] rev 12022
HOLCF: proper rep_datatype lift (see theory Lift); use plain induct_tac
instead of lift.induct_tac, use UU instead of Undef in cases;
wenzelm [Fri, 02 Nov 2001 22:02:41 +0100] rev 12021
declare transitive;
wenzelm [Fri, 02 Nov 2001 22:01:58 +0100] rev 12020
theory Calculation move to Set;
wenzelm [Fri, 02 Nov 2001 22:01:07 +0100] rev 12019
transitive declared in Pure;
paulson [Fri, 02 Nov 2001 17:55:24 +0100] rev 12018
Numerals and simprocs for types real and hypreal. The abstract
constants 0, 1 and binary numerals work harmoniously.
wenzelm [Thu, 01 Nov 2001 21:12:13 +0100] rev 12017
Goals.add_locale;
wenzelm [Thu, 01 Nov 2001 21:11:52 +0100] rev 12016
fix_frees;
improved export_def: handle args on lhs;
wenzelm [Thu, 01 Nov 2001 21:11:17 +0100] rev 12015
theorem: locale argument;
wenzelm [Thu, 01 Nov 2001 21:10:47 +0100] rev 12014
beginnings of new locales (not yet functional);
wenzelm [Thu, 01 Nov 2001 21:10:13 +0100] rev 12013
Goals.setup;
wenzelm [Thu, 01 Nov 2001 21:09:53 +0100] rev 12012
parking code for old-style locales here;
wenzelm [Wed, 31 Oct 2001 22:05:37 +0100] rev 12011
tuned notation (degree instead of dollar);
wenzelm [Wed, 31 Oct 2001 22:04:29 +0100] rev 12010
theorem(_i): locale argument;
contexts 0 and 1 in state now refer to theory and locale, respectively;
unified export (no longer uses global "standard");
wenzelm [Wed, 31 Oct 2001 22:02:33 +0100] rev 12009
Proof.init_state thy None;
wenzelm [Wed, 31 Oct 2001 22:02:11 +0100] rev 12008
simplified export;
tuned printing of fixes;
wenzelm [Wed, 31 Oct 2001 22:00:25 +0100] rev 12007
'atomize': CHANGED_PROP;
wenzelm [Wed, 31 Oct 2001 22:00:02 +0100] rev 12006
global statements: locale argument;
wenzelm [Wed, 31 Oct 2001 21:59:25 +0100] rev 12005
added local_standard;
wenzelm [Wed, 31 Oct 2001 21:59:07 +0100] rev 12004
IsarThy.theorem_i: no locale;
wenzelm [Wed, 31 Oct 2001 21:58:04 +0100] rev 12003
removed obsolete (rule equal_intr_rule);
berghofe [Wed, 31 Oct 2001 20:00:35 +0100] rev 12002
Additional rules for simplifying inside "Goal"
berghofe [Wed, 31 Oct 2001 19:59:21 +0100] rev 12001
- Tuned add_cnstrt
- Fixed bug in reconstruct_proof that caused infinite loop
berghofe [Wed, 31 Oct 2001 19:49:36 +0100] rev 12000
Removed name_thm from finish_global.
berghofe [Wed, 31 Oct 2001 19:41:29 +0100] rev 11999
Tuned function thm_proof.
berghofe [Wed, 31 Oct 2001 19:37:04 +0100] rev 11998
- enter_thmx -> enter_thms
- improved naming of theorems: enter_thms now takes functions pre_name and post_name
as arguments
berghofe [Wed, 31 Oct 2001 19:32:05 +0100] rev 11997
norm_hhf_eq is now stored using open_store_standard_thm.
wenzelm [Wed, 31 Oct 2001 01:28:39 +0100] rev 11996
induct: internalize ``missing'' consumes-facts from goal state
(enables unstructured scripts to perform elim-style induction);
wenzelm [Wed, 31 Oct 2001 01:27:04 +0100] rev 11995
- 'induct' may now use elim-style induction rules without chaining
facts, using ``missing'' premises from the goal state; this allows
rules stemming from inductive sets to be applied in unstructured
scripts, while still benefitting from proper handling of non-atomic
statements; NB: major inductive premises need to be put first, all the
rest of the goal is passed through the induction;
wenzelm [Wed, 31 Oct 2001 01:26:42 +0100] rev 11994
(induct set: ...);
wenzelm [Wed, 31 Oct 2001 01:22:27 +0100] rev 11993
put_consumes: really overwrite existing tag;
wenzelm [Wed, 31 Oct 2001 01:21:56 +0100] rev 11992
finish_global: Tactic.norm_hhf;
wenzelm [Wed, 31 Oct 2001 01:21:31 +0100] rev 11991
use HOL.induct_XXX;
wenzelm [Wed, 31 Oct 2001 01:21:01 +0100] rev 11990
use induct_rulify2;
wenzelm [Wed, 31 Oct 2001 01:20:42 +0100] rev 11989
renamed inductive_XXX to induct_XXX;
added induct_impliesI;
wenzelm [Wed, 31 Oct 2001 01:19:58 +0100] rev 11988
induct_impliesI;
wenzelm [Tue, 30 Oct 2001 17:37:25 +0100] rev 11987
tuned induct proofs;
wenzelm [Tue, 30 Oct 2001 17:33:56 +0100] rev 11986
- 'induct' method now derives symbolic cases from the *rulified* rule
(before it used to rulify cases stemming from the internal atomized
version); this means that the context of a non-atomic statement
becomes is included in the hypothesis, avoiding the slightly
cumbersome show "PROP ?case" form;
wenzelm [Tue, 30 Oct 2001 17:33:03 +0100] rev 11985
tuned;
wenzelm [Tue, 30 Oct 2001 17:30:21 +0100] rev 11984
induct: cases are extracted from rulified rule;
wenzelm [Tue, 30 Oct 2001 17:29:43 +0100] rev 11983
removed obsolete make_raw;
wenzelm [Tue, 30 Oct 2001 13:43:26 +0100] rev 11982
lemma Least_mono moved from Typedef.thy to Set.thy;
wenzelm [Mon, 29 Oct 2001 17:22:18 +0100] rev 11981
tuned;
wenzelm [Mon, 29 Oct 2001 14:09:10 +0100] rev 11980
removed option -depend (not available everywhere?);
wenzelm [Sun, 28 Oct 2001 22:59:12 +0100] rev 11979
converted theory "Set";
wenzelm [Sun, 28 Oct 2001 22:58:39 +0100] rev 11978
fixed string_of_mixfix;
wenzelm [Sun, 28 Oct 2001 21:14:56 +0100] rev 11977
tuned declaration of rules;
wenzelm [Sun, 28 Oct 2001 21:10:47 +0100] rev 11976
equal_intr_rule already declared in Pure;
wenzelm [Sun, 28 Oct 2001 19:44:58 +0100] rev 11975
rules for meta-level conjunction;
wenzelm [Sun, 28 Oct 2001 19:44:26 +0100] rev 11974
tuned prove;
wenzelm [Sat, 27 Oct 2001 23:21:19 +0200] rev 11973
tuned;
wenzelm [Sat, 27 Oct 2001 23:19:55 +0200] rev 11972
added prove;
wenzelm [Sat, 27 Oct 2001 23:19:37 +0200] rev 11971
declare equal_intr_rule as intro;
wenzelm [Sat, 27 Oct 2001 23:19:04 +0200] rev 11970
tuned prove;
added prove_standard;
wenzelm [Sat, 27 Oct 2001 23:18:40 +0200] rev 11969
removed obsolete goal_subclass, goal_arity;
wenzelm [Sat, 27 Oct 2001 23:17:46 +0200] rev 11968
use Tactic.prove;
wenzelm [Sat, 27 Oct 2001 23:17:28 +0200] rev 11967
use Tactic.prove;
improved proof of equality rule;
wenzelm [Sat, 27 Oct 2001 23:16:15 +0200] rev 11966
tuned;
wenzelm [Sat, 27 Oct 2001 23:15:52 +0200] rev 11965
* Pure/axclass: removed obsolete ML interface goal_subclass/goal_arity;
wenzelm [Sat, 27 Oct 2001 23:13:42 +0200] rev 11964
updated;
wenzelm [Sat, 27 Oct 2001 00:09:59 +0200] rev 11963
impose hyps on initial goal configuration (prevents res_inst_tac problems);
wenzelm [Sat, 27 Oct 2001 00:07:48 +0200] rev 11962
added "atomize" method;
wenzelm [Sat, 27 Oct 2001 00:07:19 +0200] rev 11961
prove: primitive goal interface for internal use;
wenzelm [Sat, 27 Oct 2001 00:06:46 +0200] rev 11960
added impose_hyps;
wenzelm [Sat, 27 Oct 2001 00:06:22 +0200] rev 11959
exclude field_simps from user-level "simps";
wenzelm [Sat, 27 Oct 2001 00:05:50 +0200] rev 11958
Isar: fixed rep_datatype args;
wenzelm [Sat, 27 Oct 2001 00:05:14 +0200] rev 11957
hardwire qualified const names;
wenzelm [Sat, 27 Oct 2001 00:00:55 +0200] rev 11956
removed "more" class;
wenzelm [Sat, 27 Oct 2001 00:00:38 +0200] rev 11955
moved product cases/induct to theory Datatype;
wenzelm [Sat, 27 Oct 2001 00:00:05 +0200] rev 11954
made new-style theory;
tuned;
wenzelm [Fri, 26 Oct 2001 23:59:13 +0200] rev 11953
atomize_conj;
wenzelm [Fri, 26 Oct 2001 23:58:21 +0200] rev 11952
* Pure: method 'atomize' presents local goal premises as object-level
statements (atomic meta-level propositions); setup controlled via
rewrite rules declarations of 'atomize' attribute; example
application: 'induct' method with proper rule statements in improper
proof *scripts*;
berghofe [Fri, 26 Oct 2001 23:17:49 +0200] rev 11951
Fixed several bugs concerning arbitrarily branching datatypes.
berghofe [Fri, 26 Oct 2001 19:06:53 +0200] rev 11950
Eliminated occurrence of rule_format.
wenzelm [Fri, 26 Oct 2001 18:16:45 +0200] rev 11949
tuned;
wenzelm [Fri, 26 Oct 2001 18:16:31 +0200] rev 11948
need at least 3 latex runs to get toc right!
wenzelm [Fri, 26 Oct 2001 16:49:10 +0200] rev 11947
tuned;
wenzelm [Fri, 26 Oct 2001 16:18:14 +0200] rev 11946
tuned;
wenzelm [Fri, 26 Oct 2001 14:22:33 +0200] rev 11945
Rrightarrow;
wenzelm [Fri, 26 Oct 2001 14:02:58 +0200] rev 11944
tuned notation;
wenzelm [Fri, 26 Oct 2001 12:24:19 +0200] rev 11943
tuned notation;
wenzelm [Thu, 25 Oct 2001 22:59:11 +0200] rev 11942
accomodate some recent changes of record package;
wenzelm [Thu, 25 Oct 2001 22:58:26 +0200] rev 11941
updated;
wenzelm [Thu, 25 Oct 2001 22:43:58 +0200] rev 11940
removed "more" sort;
refer to properly named theorems internally;
wenzelm [Thu, 25 Oct 2001 22:43:05 +0200] rev 11939
updated records;
wenzelm [Thu, 25 Oct 2001 22:42:50 +0200] rev 11938
'simplified' att: args;
wenzelm [Thu, 25 Oct 2001 22:42:12 +0200] rev 11937
* HOL/record:
- removed "more" class (simply use "term") -- INCOMPATIBILITY;
wenzelm [Thu, 25 Oct 2001 22:41:07 +0200] rev 11936
* Provers: 'simplified' attribute may refer to explicit rules instead
of full simplifier context; 'iff' attribute handles conditional rules;
* HOL/record:
- provides cases/induct rules for use with corresponding Isar methods;
- old "make" and "make_scheme" operation removed -- INCOMPATIBILITY;
- new derived operations "make" (for adding fields of current
record), "extend" to promote fixed record to record scheme, and
"truncate" for the reverse; cf. theorems "derived_defs", which are
*not* declared as simp by default;
- internal definitions directly based on a light-weight abstract
theory of product types over typedef rather than datatype;
berghofe [Thu, 25 Oct 2001 20:04:43 +0200] rev 11935
Replaced main proof by proper Isar script.
wenzelm [Thu, 25 Oct 2001 20:00:11 +0200] rev 11934
derived operations are now: make, extend, truncate (cf. derived_defs);
wenzelm [Thu, 25 Oct 2001 19:59:00 +0200] rev 11933
tuned;
wenzelm [Thu, 25 Oct 2001 19:55:41 +0200] rev 11932
check_goal: setmp proofs 0;
kleing [Thu, 25 Oct 2001 16:09:39 +0200] rev 11931
added windowlistener (can now close the frame by window controls)
wenzelm [Thu, 25 Oct 2001 02:13:02 +0200] rev 11930
* HOL/record:
- provides cases/induct rules for use with corresponding Isar methods;
- "record" operation truncates to particular fixed record (acts like
a type cast);
- make_defs no longer part of default simps;
- internal definitions directly based on a light-weight abstract
theory of product types over typedef rather than datatype;
wenzelm [Thu, 25 Oct 2001 02:12:10 +0200] rev 11929
innermost_params;
wenzelm [Thu, 25 Oct 2001 02:11:49 +0200] rev 11928
(simp add: point.make_def);
wenzelm [Thu, 25 Oct 2001 02:11:28 +0200] rev 11927
provodes induct/cases for use with corresponding Isar methods;
"record" operation (acts as type cast);
internal field_inducts, field_cases;
make_defs no longer declared as simps;
fixed printing of fixed records;
wenzelm [Wed, 24 Oct 2001 19:20:02 +0200] rev 11926
further 1.73 changes: added fix_direct, simplified assume interface;
wenzelm [Wed, 24 Oct 2001 19:18:23 +0200] rev 11925
added read_prop_schematic;
wenzelm [Wed, 24 Oct 2001 19:18:10 +0200] rev 11924
simplified ProofContext.assume interface;
wenzelm [Wed, 24 Oct 2001 17:38:29 +0200] rev 11923
moved lambda to Pure/term.ML;
wenzelm [Wed, 24 Oct 2001 17:38:19 +0200] rev 11922
added lambda;
wenzelm [Wed, 24 Oct 2001 17:37:58 +0200] rev 11921
* clasimp: ``iff'' declarations now handle conditional rules as well;
wenzelm [Wed, 24 Oct 2001 17:31:58 +0200] rev 11920
added string_of_mixfix;
wenzelm [Wed, 24 Oct 2001 17:31:20 +0200] rev 11919
print_depth 8 from the very beginning;
wenzelm [Tue, 23 Oct 2001 23:29:29 +0200] rev 11918
added export_assume, export_presume, export_def (from proof.ML);
wenzelm [Tue, 23 Oct 2001 23:28:59 +0200] rev 11917
moved RANGE to tctical.ML;
moved export_assume, export_presume, export_def to proof_context.ML;
wenzelm [Tue, 23 Oct 2001 23:28:01 +0200] rev 11916
added RANGE (from Isar/proof.ML);
wenzelm [Tue, 23 Oct 2001 22:59:14 +0200] rev 11915
print fixed names as plain strings;
wenzelm [Tue, 23 Oct 2001 22:58:15 +0200] rev 11914
eliminated old numerals;
wenzelm [Tue, 23 Oct 2001 22:57:52 +0200] rev 11913
use generic 1 instead of Numeral1;
use improved iff declaration;
tuned;
wenzelm [Tue, 23 Oct 2001 22:56:55 +0200] rev 11912
eliminated Numeral0;
wenzelm [Tue, 23 Oct 2001 22:54:01 +0200] rev 11911
build option enables most basic browser info (for proper recording of session);
wenzelm [Tue, 23 Oct 2001 22:53:08 +0200] rev 11910
build option;
wenzelm [Tue, 23 Oct 2001 22:52:45 +0200] rev 11909
tuned;
wenzelm [Tue, 23 Oct 2001 22:52:31 +0200] rev 11908
eliminated old numerals;
wenzelm [Tue, 23 Oct 2001 22:51:30 +0200] rev 11907
pass build mode to process;
wenzelm [Tue, 23 Oct 2001 19:15:00 +0200] rev 11906
removed export_thm;
wenzelm [Tue, 23 Oct 2001 19:14:47 +0200] rev 11905
trace_rules: only non-empty;
wenzelm [Tue, 23 Oct 2001 19:14:31 +0200] rev 11904
removed obsolete "exported" att;
wenzelm [Tue, 23 Oct 2001 19:14:13 +0200] rev 11903
replace_dummy_patterns: lift over bounds;
wenzelm [Tue, 23 Oct 2001 19:13:44 +0200] rev 11902
iff: always rotate prems;
wenzelm [Tue, 23 Oct 2001 19:13:17 +0200] rev 11901
apply(simp add: three_def numerals) (* FIXME !? *);
wenzelm [Tue, 23 Oct 2001 19:12:58 +0200] rev 11900
unset DISPLAY (again);
wenzelm [Tue, 23 Oct 2001 19:12:37 +0200] rev 11899
* Pure: removed obsolete 'exported' attribute;
* Pure: dummy pattern "_" in is/let is now automatically ``lifted''
over bound variables: "ALL x. P x --> Q x" (is "ALL x. _ --> ?C x")
supersedes more cumbersome ... (is "ALL x. _ x --> ?C x");
wenzelm [Mon, 22 Oct 2001 23:39:00 +0200] rev 11898
*** empty log message ***
wenzelm [Mon, 22 Oct 2001 18:07:53 +0200] rev 11897
moved object_logic.ML to Isar/object_logic.ML;
wenzelm [Mon, 22 Oct 2001 18:07:30 +0200] rev 11896
moved locale.ML to Isar/locale.ML;
wenzelm [Mon, 22 Oct 2001 18:04:26 +0200] rev 11895
moved goal related stuff to goals.ML;
wenzelm [Mon, 22 Oct 2001 18:04:11 +0200] rev 11894
Display.current_goals_markers;
wenzelm [Mon, 22 Oct 2001 18:04:00 +0200] rev 11893
tuned;
wenzelm [Mon, 22 Oct 2001 18:03:49 +0200] rev 11892
moved prove_goalw_cterm to goals.ML;
cleaned up;
wenzelm [Mon, 22 Oct 2001 18:03:21 +0200] rev 11891
moved local defs to proof.ML (for locales);
wenzelm [Mon, 22 Oct 2001 18:02:50 +0200] rev 11890
improved source arrangement of obtain;
wenzelm [Mon, 22 Oct 2001 18:02:21 +0200] rev 11889
rearrange sources for locales;
wenzelm [Mon, 22 Oct 2001 18:02:04 +0200] rev 11888
Display.print_current_goals_fn;
wenzelm [Mon, 22 Oct 2001 18:01:52 +0200] rev 11887
Display.print_goals;
wenzelm [Mon, 22 Oct 2001 18:01:38 +0200] rev 11886
Display.pretty_thms;
wenzelm [Mon, 22 Oct 2001 18:01:26 +0200] rev 11885
qualified names;
wenzelm [Mon, 22 Oct 2001 18:01:15 +0200] rev 11884
make this module appeat late in Pure;
moved print_current_goals to display.ML;
added quick_and_dirty_prove_goalw_cterm (from Isar/skip_proof.ML);
added thm database functions (from Thy/thm_database.ML);
wenzelm [Mon, 22 Oct 2001 17:59:39 +0200] rev 11883
print_goals stuff is back (from locale.ML);
wenzelm [Mon, 22 Oct 2001 17:58:56 +0200] rev 11882
reorganize sources to accomodate locales;
wenzelm [Mon, 22 Oct 2001 17:58:37 +0200] rev 11881
corollary;
wenzelm [Mon, 22 Oct 2001 17:58:26 +0200] rev 11880
quick_and_dirty_prove_goalw_cterm;
wenzelm [Mon, 22 Oct 2001 17:58:11 +0200] rev 11879
javac -depend;
wenzelm [Mon, 22 Oct 2001 17:56:16 +0200] rev 11878
-D generated;
berghofe [Mon, 22 Oct 2001 14:58:05 +0200] rev 11877
Added "clean" target.
berghofe [Mon, 22 Oct 2001 14:55:16 +0200] rev 11876
Fixed problem with batch mode layout, which caused an AWT exception when
no X11 connection was available.
berghofe [Mon, 22 Oct 2001 14:53:52 +0200] rev 11875
initBrowser now has additional noAWT argument.
berghofe [Mon, 22 Oct 2001 14:52:43 +0200] rev 11874
Constructor no longer takes font as an argument.
berghofe [Mon, 22 Oct 2001 14:52:12 +0200] rev 11873
Moved font settings from TreeNode to TreeBrowser.
berghofe [Mon, 22 Oct 2001 14:51:39 +0200] rev 11872
Moved font settings from Vertex to GraphView.
paulson [Mon, 22 Oct 2001 12:11:00 +0200] rev 11871
deleted the redundant first argument of adjust(a,b)
paulson [Mon, 22 Oct 2001 12:01:35 +0200] rev 11870
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
to their abstract counterparts, while other binary numerals work correctly.
paulson [Mon, 22 Oct 2001 11:55:35 +0200] rev 11869
New simproc, needed to cope with combinations of (abstract) 0, (abstract) 1,
binary numerals in literal arithmetic.
paulson [Mon, 22 Oct 2001 11:54:22 +0200] rev 11868
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
to their abstract counterparts, while other binary numerals work correctly.
wenzelm [Mon, 22 Oct 2001 11:01:30 +0200] rev 11867
keep DISPLAY;
wenzelm [Sun, 21 Oct 2001 19:49:29 +0200] rev 11866
updated;
wenzelm [Sun, 21 Oct 2001 19:48:19 +0200] rev 11865
renamed to Typedefs.thy to avoid conflict with main HOL version;
wenzelm [Sun, 21 Oct 2001 19:44:25 +0200] rev 11864
* proper spacing of consecutive markup elements, especially text
blocks after section headings;
wenzelm [Sun, 21 Oct 2001 19:42:53 +0200] rev 11863
\newif\ifisamarkup controls spacing of isabeginpar;
wenzelm [Sun, 21 Oct 2001 19:42:24 +0200] rev 11862
improved spacing;
wenzelm [Sun, 21 Oct 2001 19:41:43 +0200] rev 11861
maintain Latex.flag_markup;
wenzelm [Sun, 21 Oct 2001 19:40:39 +0200] rev 11860
flag_markup;
wenzelm [Sun, 21 Oct 2001 19:36:12 +0200] rev 11859
Types/document/Typedefs;
wenzelm [Sun, 21 Oct 2001 19:35:40 +0200] rev 11858
renamed Typedef.thy to Typedefs.thy (former already present in main HOL);
wenzelm [Sat, 20 Oct 2001 22:07:44 +0200] rev 11857
got rid of separate root.tex;
wenzelm [Sat, 20 Oct 2001 20:23:37 +0200] rev 11856
graceful interpretation of -i/-d/-D options;
verbose: additional messages/warnings;
include document graph;
wenzelm [Sat, 20 Oct 2001 20:22:17 +0200] rev 11855
include document graph;
wenzelm [Sat, 20 Oct 2001 20:21:40 +0200] rev 11854
document graph option;
wenzelm [Sat, 20 Oct 2001 20:21:14 +0200] rev 11853
conditional: bool -> (unit -> unit) -> unit;
std_error: string -> unit;
wenzelm [Sat, 20 Oct 2001 20:20:41 +0200] rev 11852
added TextIO.stdErr;
wenzelm [Sat, 20 Oct 2001 20:20:21 +0200] rev 11851
include document graph;
tuned;
wenzelm [Sat, 20 Oct 2001 20:19:47 +0200] rev 11850
document graphs for several sessions;
wenzelm [Sat, 20 Oct 2001 20:18:57 +0200] rev 11849
tuned;
wenzelm [Sat, 20 Oct 2001 20:18:45 +0200] rev 11848
calculational rules moved from FOL to IFOL;
wenzelm [Sat, 20 Oct 2001 20:18:19 +0200] rev 11847
option -g for document graph;
removed all presumptions about -d/-D (handled by isabelle process);
wenzelm [Sat, 20 Oct 2001 20:16:55 +0200] rev 11846
option -q also excludes -v true in generated stuff;
tuned message;
wenzelm [Sat, 20 Oct 2001 20:15:44 +0200] rev 11845
dvips -q;
wenzelm [Sat, 20 Oct 2001 20:15:27 +0200] rev 11844
removed -v option (handled by isabelle process);
wenzelm [Sat, 20 Oct 2001 20:14:56 +0200] rev 11843
-o pdf: produce *both* eps and pdf;
tuned;
wenzelm [Sat, 20 Oct 2001 20:14:16 +0200] rev 11842
* greatly simplified document preparation setup, including more
graceful interpretation of isatool usedir -i/-d/-D options, and more
instructive isatool mkdir; users should basically be able to get
started with "isatool mkdir Test && isatool make";
* theory dependency graph may now be incorporated into documents;
isatool usedir -g true will produce session_graph.eps/.pdf for use
with \includegraphics of LaTeX;
wenzelm [Fri, 19 Oct 2001 22:03:25 +0200] rev 11841
got rid of ML proof scripts;
wenzelm [Fri, 19 Oct 2001 22:02:25 +0200] rev 11840
induct_method.ML -- proof by cases and induction on sets and types (Isar);
wenzelm [Fri, 19 Oct 2001 22:02:02 +0200] rev 11839
latex output: bold lambda;
wenzelm [Fri, 19 Oct 2001 22:01:25 +0200] rev 11838
got rid of ML proof scripts for Product_Type;
wenzelm [Fri, 19 Oct 2001 22:00:08 +0200] rev 11837
got rid of Provers/split_paired_all.ML;
wenzelm [Fri, 19 Oct 2001 21:59:33 +0200] rev 11836
improved default dependencies;
wenzelm [Fri, 19 Oct 2001 12:17:04 +0200] rev 11835
revert to proper version (!);
wenzelm [Thu, 18 Oct 2001 21:27:47 +0200] rev 11834
GPLed;
wenzelm [Thu, 18 Oct 2001 21:22:40 +0200] rev 11833
tuned;
wenzelm [Thu, 18 Oct 2001 21:07:29 +0200] rev 11832
use abstract product type instead of datatype;
wenzelm [Thu, 18 Oct 2001 21:05:35 +0200] rev 11831
moved atomize stuff to theory HOL;
wenzelm [Thu, 18 Oct 2001 21:03:43 +0200] rev 11830
legacy interfaces for axclass instantiation;
wenzelm [Thu, 18 Oct 2001 21:02:46 +0200] rev 11829
added map_base;
wenzelm [Thu, 18 Oct 2001 21:02:26 +0200] rev 11828
sane internal interfaces for instance;
wenzelm [Thu, 18 Oct 2001 21:01:59 +0200] rev 11827
sane internal interface for add_typedef(_i);
wenzelm [Thu, 18 Oct 2001 21:01:18 +0200] rev 11826
proper setup for abstract product types;
wenzelm [Thu, 18 Oct 2001 20:59:59 +0200] rev 11825
moved InductMethod.setup to theory HOL;
wenzelm [Thu, 18 Oct 2001 20:59:33 +0200] rev 11824
setup generic cases and induction (from Inductive.thy);
wenzelm [Wed, 17 Oct 2001 20:25:51 +0200] rev 11823
guillemot syntax;
wenzelm [Wed, 17 Oct 2001 20:25:19 +0200] rev 11822
improved internal interface of typedef;
wenzelm [Wed, 17 Oct 2001 20:24:37 +0200] rev 11821
abstract product types;
wenzelm [Wed, 17 Oct 2001 20:24:03 +0200] rev 11820
proper proof of split_paired_all (presently unused);
wenzelm [Wed, 17 Oct 2001 18:52:30 +0200] rev 11819
tuned comments;
wenzelm [Wed, 17 Oct 2001 18:51:03 +0200] rev 11818
added mk_UNIV;
wenzelm [Wed, 17 Oct 2001 18:50:49 +0200] rev 11817
tuned;
wenzelm [Tue, 16 Oct 2001 23:02:14 +0200] rev 11816
simplified exporter interface;
wenzelm [Tue, 16 Oct 2001 23:00:21 +0200] rev 11815
added implies_intr_goals;
wenzelm [Tue, 16 Oct 2001 22:59:30 +0200] rev 11814
tuned;
berghofe [Tue, 16 Oct 2001 19:56:31 +0200] rev 11813
Tuned.
berghofe [Tue, 16 Oct 2001 19:54:53 +0200] rev 11812
Removed exit command from end of main method.
berghofe [Tue, 16 Oct 2001 19:54:24 +0200] rev 11811
PS method now calculates layout using default font metrics.
berghofe [Tue, 16 Oct 2001 19:53:12 +0200] rev 11810
Inserted table for character widths.
wenzelm [Tue, 16 Oct 2001 17:58:13 +0200] rev 11809
tuned induction proofs;
wenzelm [Tue, 16 Oct 2001 17:56:12 +0200] rev 11808
dest_env: norm_term on rhs;
wenzelm [Tue, 16 Oct 2001 17:55:53 +0200] rev 11807
typedef: export result;
wenzelm [Tue, 16 Oct 2001 17:55:38 +0200] rev 11806
ignore typedef result;
wenzelm [Tue, 16 Oct 2001 17:55:16 +0200] rev 11805
declare projected induction rules stemming from nested recursion;
wenzelm [Tue, 16 Oct 2001 17:52:07 +0200] rev 11804
TypedefPackage.add_typedef_no_result;
wenzelm [Tue, 16 Oct 2001 17:51:50 +0200] rev 11803
tuned;
wenzelm [Tue, 16 Oct 2001 17:51:12 +0200] rev 11802
* HOL: concrete setsum syntax "\<Sum>i:A. b" == "setsum (%i. b) A"
(beware of argument permutation!);
wenzelm [Tue, 16 Oct 2001 17:25:44 +0200] rev 11801
option -o FILE --output to FILE (ps, eps, pdf);
wenzelm [Tue, 16 Oct 2001 17:24:33 +0200] rev 11800
ISABELLE_EPSTOPDF="epstopdf";
berghofe [Tue, 16 Oct 2001 16:48:30 +0200] rev 11799
Font metrics used for batch mode layout (without X11 connection).
berghofe [Tue, 16 Oct 2001 16:47:54 +0200] rev 11798
Added support for batch mode layout (without X11 connection).
wenzelm [Tue, 16 Oct 2001 00:50:23 +0200] rev 11797
tuned;
wenzelm [Tue, 16 Oct 2001 00:39:34 +0200] rev 11796
improved induct;
wenzelm [Tue, 16 Oct 2001 00:35:30 +0200] rev 11795
be more careful about token class markers;
wenzelm [Tue, 16 Oct 2001 00:35:03 +0200] rev 11794
proper order of kind names;
wenzelm [Tue, 16 Oct 2001 00:34:34 +0200] rev 11793
support impromptu terminology of cases parameters;
wenzelm [Tue, 16 Oct 2001 00:33:22 +0200] rev 11792
parser for underscore (actually a symbolic identifier!);
wenzelm [Tue, 16 Oct 2001 00:32:34 +0200] rev 11791
allow empty set/type name;
wenzelm [Tue, 16 Oct 2001 00:32:01 +0200] rev 11790
simplified resolveq_cases_tac for cases, separate version for induct;
divinate instantiation of induct rules;
tuned;
wenzelm [Tue, 16 Oct 2001 00:30:53 +0200] rev 11789
tuned;
kleing [Mon, 15 Oct 2001 21:04:46 +0200] rev 11788
canonical 'cases'/'induct' rules for n-tuples (n=3..7)
kleing [Mon, 15 Oct 2001 21:04:32 +0200] rev 11787
canonical 'cases'/'induct' rules for n-tuples (n=3..7)
(really belongs to theory Product_Type, but doesn't work there yet)
wenzelm [Mon, 15 Oct 2001 20:42:06 +0200] rev 11786
setsum syntax;
wenzelm [Mon, 15 Oct 2001 20:41:14 +0200] rev 11785
intro! and elim! rules;
wenzelm [Mon, 15 Oct 2001 20:36:48 +0200] rev 11784
tuned NetRules;
wenzelm [Mon, 15 Oct 2001 20:36:04 +0200] rev 11783
Tactic.orderlist;
wenzelm [Mon, 15 Oct 2001 20:35:42 +0200] rev 11782
ObjectLogic.rulify;
wenzelm [Mon, 15 Oct 2001 20:35:10 +0200] rev 11781
Tactic.rewrite_cterm;
wenzelm [Mon, 15 Oct 2001 20:34:44 +0200] rev 11780
GPLed;
wenzelm [Mon, 15 Oct 2001 20:34:26 +0200] rev 11779
ring instead of ringS;
wenzelm [Mon, 15 Oct 2001 20:34:12 +0200] rev 11778
ring includes plus_ac0;
wenzelm [Mon, 15 Oct 2001 20:33:42 +0200] rev 11777
tuned;
wenzelm [Mon, 15 Oct 2001 20:33:05 +0200] rev 11776
support weight;
wenzelm [Mon, 15 Oct 2001 20:32:13 +0200] rev 11775
bang_args;
wenzelm [Mon, 15 Oct 2001 20:31:52 +0200] rev 11774
qualify some names;
wenzelm [Mon, 15 Oct 2001 20:31:18 +0200] rev 11773
map_nth_elem;
oheimb [Mon, 15 Oct 2001 17:02:57 +0200] rev 11772
renamed reset_locs to del_locs
wenzelm [Sun, 14 Oct 2001 22:15:07 +0200] rev 11771
moved rulify to ObjectLogic;
wenzelm [Sun, 14 Oct 2001 22:08:29 +0200] rev 11770
moved rulify to ObjectLogic;
wenzelm [Sun, 14 Oct 2001 22:07:01 +0200] rev 11769
added qed_spec_mp etc.;
wenzelm [Sun, 14 Oct 2001 22:05:46 +0200] rev 11768
unified rewrite/rewrite_cterm/simplify interface;
wenzelm [Sun, 14 Oct 2001 22:05:01 +0200] rev 11767
tuned rewrite/simplify interface;
wenzelm [Sun, 14 Oct 2001 20:10:44 +0200] rev 11766
improved atomize setup;
wenzelm [Sun, 14 Oct 2001 20:09:59 +0200] rev 11765
atomize_tac etc. moved to object_logic.ML;
wenzelm [Sun, 14 Oct 2001 20:09:19 +0200] rev 11764
use ObjectLogic;
wenzelm [Sun, 14 Oct 2001 20:09:05 +0200] rev 11763
added 'atomize' attribute;
wenzelm [Sun, 14 Oct 2001 20:08:42 +0200] rev 11762
tuned full_rewrite;
wenzelm [Sun, 14 Oct 2001 20:08:26 +0200] rev 11761
ObjectLogic.setup;
wenzelm [Sun, 14 Oct 2001 20:08:11 +0200] rev 11760
tuned;
wenzelm [Sun, 14 Oct 2001 20:07:32 +0200] rev 11759
added object_logic.ML;
wenzelm [Sun, 14 Oct 2001 20:07:11 +0200] rev 11758
fixed auto steps (due to changed atomize);
wenzelm [Sun, 14 Oct 2001 20:06:13 +0200] rev 11757
Specifics about common object-logics.
wenzelm [Sun, 14 Oct 2001 20:05:42 +0200] rev 11756
use ObjectLogic stuff;
wenzelm [Sun, 14 Oct 2001 20:05:07 +0200] rev 11755
"HOL.mono";
wenzelm [Sun, 14 Oct 2001 20:04:05 +0200] rev 11754
ObjectLogic.atomize_tac;
wenzelm [Sun, 14 Oct 2001 20:02:59 +0200] rev 11753
improved atomize setup;
wenzelm [Sun, 14 Oct 2001 20:02:30 +0200] rev 11752
removed Ord;
wenzelm [Sun, 14 Oct 2001 20:02:11 +0200] rev 11751
removed Ord.thy (now part of HOL.thy).
wenzelm [Sun, 14 Oct 2001 20:01:42 +0200] rev 11750
judgment Trueprop;
proper declarations of atomize rules;
incorporate theory Ord;
proper section and text markup;
tuned;
wenzelm [Sun, 14 Oct 2001 20:00:32 +0200] rev 11749
added ML bindings from former theory Ord;
wenzelm [Sun, 14 Oct 2001 19:59:55 +0200] rev 11748
eliminated atomize rules;
wenzelm [Sun, 14 Oct 2001 19:59:15 +0200] rev 11747
judgment Trueprop;
proper declarations of atomize rules;
wenzelm [Sat, 13 Oct 2001 21:46:53 +0200] rev 11746
updated;
wenzelm [Sat, 13 Oct 2001 21:45:23 +0200] rev 11745
* HOL: 'typedef' now allows alternative names for Rep/Abs morphisms;
wenzelm [Sat, 13 Oct 2001 21:44:58 +0200] rev 11744
'morphisms' spec;
tuned goal pattern for set;
wenzelm [Sat, 13 Oct 2001 21:43:00 +0200] rev 11743
tuned;
wenzelm [Sat, 13 Oct 2001 20:32:38 +0200] rev 11742
generic theorem kinds;
wenzelm [Sat, 13 Oct 2001 20:32:07 +0200] rev 11741
generic theorem kinds ("theorem", "lemma" etc.);
wenzelm [Sat, 13 Oct 2001 20:31:34 +0200] rev 11740
IsarThy.theorem_i Drule.internalK;
wenzelm [Sat, 13 Oct 2001 20:31:05 +0200] rev 11739
Drule.tag_internal;
wenzelm [Sat, 13 Oct 2001 20:30:38 +0200] rev 11738
* Pure: added 'corollary' command;
berghofe [Fri, 12 Oct 2001 18:29:51 +0200] rev 11737
Tuned comment.
berghofe [Fri, 12 Oct 2001 16:57:07 +0200] rev 11736
- Exported goals_conv and fconv_rule
- Added forall_conv
wenzelm [Fri, 12 Oct 2001 12:13:31 +0200] rev 11735
removed vars_of, concls_of;
removed additional rule instantiation argument;
proper enumeration of type rules;
append possibilities of set and type rules (analogous to elim-intro in 'rule');
wenzelm [Fri, 12 Oct 2001 12:11:39 +0200] rev 11734
declare impE iffD1 iffD2 ad elim of Pure;
wenzelm [Fri, 12 Oct 2001 12:10:07 +0200] rev 11733
removed lookups count;
always try headless rules;
wenzelm [Fri, 12 Oct 2001 12:09:38 +0200] rev 11732
added make_thm (sort-of);
wenzelm [Fri, 12 Oct 2001 12:09:21 +0200] rev 11731
added trace_rules, trace;
wenzelm [Fri, 12 Oct 2001 12:08:57 +0200] rev 11730
removed get_cases, get_induct;
added find_cases[ST], finde_induct[ST];
proper indexing of types;
wenzelm [Fri, 12 Oct 2001 12:08:04 +0200] rev 11729
removed read_inst', no longer export insts';
wenzelm [Fri, 12 Oct 2001 12:07:27 +0200] rev 11728
fixed typid;
wenzelm [Fri, 12 Oct 2001 12:06:54 +0200] rev 11727
test: use SkipProof.make_thm instead of Thm.assume;
wenzelm [Fri, 12 Oct 2001 12:06:23 +0200] rev 11726
tuned;
wenzelm [Fri, 12 Oct 2001 12:06:10 +0200] rev 11725
HOLogic.dest_concls, InductAttrib.vars_of;
wenzelm [Fri, 12 Oct 2001 12:05:46 +0200] rev 11724
declare impE iffD1 iffD2 as elim of Pure;
wenzelm [Fri, 12 Oct 2001 12:05:02 +0200] rev 11723
moved trace_rules to Pure/Isar/method.ML;
some_rule_tac: prefer Method.some_rule_tac of Pure, no special
handling of imp_elim;
wenzelm [Thu, 11 Oct 2001 21:25:45 +0200] rev 11722
* Isar/Pure: fixed 'token_translation' command;
wenzelm [Thu, 11 Oct 2001 19:22:15 +0200] rev 11721
added try;
wenzelm [Thu, 11 Oct 2001 19:22:00 +0200] rev 11720
added certify_tyname;
berghofe [Wed, 10 Oct 2001 18:41:13 +0200] rev 11719
Exported output_symbols.
berghofe [Wed, 10 Oct 2001 18:40:46 +0200] rev 11718
Removed unnecessary application of Drule.standard.
berghofe [Wed, 10 Oct 2001 18:39:38 +0200] rev 11717
Fixed erroneous type constraint in token_translation function.
berghofe [Wed, 10 Oct 2001 18:38:21 +0200] rev 11716
Exported output_with.
berghofe [Wed, 10 Oct 2001 18:37:52 +0200] rev 11715
Tuned several functions to improve sharing of unchanged subproofs.
wenzelm [Tue, 09 Oct 2001 18:11:07 +0200] rev 11714
added global modes ref;
wenzelm [Mon, 08 Oct 2001 15:23:20 +0200] rev 11713
sane numerals (stage 3): provide generic "1" on all number types;
wenzelm [Mon, 08 Oct 2001 14:30:28 +0200] rev 11712
* added default LaTeX bindings for \<tturnstile> and \<TTurnstile>;
note that these symbols are unavailable in Proof General / X-Symbol;
wenzelm [Mon, 08 Oct 2001 14:29:02 +0200] rev 11711
fixed numerals;
wenzelm [Mon, 08 Oct 2001 14:19:42 +0200] rev 11710
added tturnstile, TTurnstile;
wenzelm [Mon, 08 Oct 2001 14:19:22 +0200] rev 11709
*** empty log message ***
wenzelm [Mon, 08 Oct 2001 12:28:43 +0200] rev 11708
*** empty log message ***
wenzelm [Mon, 08 Oct 2001 12:27:19 +0200] rev 11707
replace 0r/1r by 0/1;
wenzelm [Mon, 08 Oct 2001 12:13:56 +0200] rev 11706
*** empty log message ***
wenzelm [Mon, 08 Oct 2001 12:13:34 +0200] rev 11705
fixed numerals;
wenzelm [Sat, 06 Oct 2001 00:02:46 +0200] rev 11704
* sane numerals (stage 2): plain "num" syntax (removed "#");
wenzelm [Fri, 05 Oct 2001 23:58:52 +0200] rev 11703
tuned;
wenzelm [Fri, 05 Oct 2001 23:58:17 +0200] rev 11702
*** empty log message ***
wenzelm [Fri, 05 Oct 2001 21:52:39 +0200] rev 11701
sane numerals (stage 1): added generic 1, removed 1' and 2 on nat,
"num" syntax (still with "#"), Numeral0, Numeral1;
wenzelm [Fri, 05 Oct 2001 21:50:37 +0200] rev 11700
*** empty log message ***
wenzelm [Fri, 05 Oct 2001 21:49:59 +0200] rev 11699
"num" syntax;
wenzelm [Fri, 05 Oct 2001 21:49:15 +0200] rev 11698
added axclass "one" and polymorphic const "1";
print consts "0" and "1" with type constraints;
wenzelm [Fri, 05 Oct 2001 21:48:04 +0200] rev 11697
added "num" token;
wenzelm [Fri, 05 Oct 2001 21:42:10 +0200] rev 11696
induct: case names;
wenzelm [Fri, 05 Oct 2001 21:37:33 +0200] rev 11695
sane spacing of "-";
wenzelm [Fri, 05 Oct 2001 16:04:56 +0200] rev 11694
tuned;
wenzelm [Thu, 04 Oct 2001 23:27:42 +0200] rev 11693
Thm.major_prem_of part of Logic.strip_assums_concl;
wenzelm [Thu, 04 Oct 2001 23:27:01 +0200] rev 11692
major_prem_of: Logic.strip_assums_concl;
wenzelm [Thu, 04 Oct 2001 16:09:12 +0200] rev 11691
induct/cases made generic, removed simplified/stripped options;
wenzelm [Thu, 04 Oct 2001 16:07:43 +0200] rev 11690
improved proof by cases and induction;
wenzelm [Thu, 04 Oct 2001 16:07:20 +0200] rev 11689
removed obsolete comment;
wenzelm [Thu, 04 Oct 2001 15:43:17 +0200] rev 11688
generic induct_method.ML;
tuned;
wenzelm [Thu, 04 Oct 2001 15:42:48 +0200] rev 11687
non-oriented infix = and ~= (output only);
added case_split (with case names);
wenzelm [Thu, 04 Oct 2001 15:41:43 +0200] rev 11686
$(SRC)/Provers/induct_method.ML replaces Tools/induct_method.ML;
wenzelm [Thu, 04 Oct 2001 15:40:52 +0200] rev 11685
use "~~/src/Provers/induct_method.ML";
wenzelm [Thu, 04 Oct 2001 15:40:31 +0200] rev 11684
removed hol_rewrite_cterm (use full_rewrite_cterm from Pure);
wenzelm [Thu, 04 Oct 2001 15:40:05 +0200] rev 11683
added dest_concls;
wenzelm [Thu, 04 Oct 2001 15:39:43 +0200] rev 11682
simp_case_tac is back again from induct_method.ML;
tuned;
wenzelm [Thu, 04 Oct 2001 15:39:00 +0200] rev 11681
made generic (see Provers/induct_method.ML);
wenzelm [Thu, 04 Oct 2001 15:29:37 +0200] rev 11680
qualify MetaSimplifier;
wenzelm [Thu, 04 Oct 2001 15:29:22 +0200] rev 11679
unsymbolized;
wenzelm [Thu, 04 Oct 2001 15:28:26 +0200] rev 11678
moved atomize stuff to theory IFOL;
added induct/cases setup;
wenzelm [Thu, 04 Oct 2001 15:28:00 +0200] rev 11677
atomize stuff from theory FOL;
tuned;
wenzelm [Thu, 04 Oct 2001 15:27:13 +0200] rev 11676
added Provers/induct_method.ML, document/root.tex, ex/Natural_Numbers.thy;
wenzelm [Thu, 04 Oct 2001 15:26:14 +0200] rev 11675
theory Natural_Numbers;
wenzelm [Thu, 04 Oct 2001 15:25:51 +0200] rev 11674
use "~~/src/Provers/induct_method.ML";
wenzelm [Thu, 04 Oct 2001 15:25:31 +0200] rev 11673
Theory of the natural numbers: Peano's axioms, primitive recursion.
(Modernized version of Larry Paulson's theory "Nat".)
wenzelm [Thu, 04 Oct 2001 15:21:47 +0200] rev 11672
full_rewrite_cterm_aux (see also tactic.ML);
no longer open MetaSimplifier;
wenzelm [Thu, 04 Oct 2001 15:21:17 +0200] rev 11671
added full_rewrite_cterm;
wenzelm [Thu, 04 Oct 2001 15:20:40 +0200] rev 11670
proof by cases and induction on types and sets (used to be specific for HOL);
wenzelm [Thu, 04 Oct 2001 15:19:56 +0200] rev 11669
qualify MetaSimplifier;
wenzelm [Thu, 04 Oct 2001 14:49:38 +0200] rev 11668
added dest_conj, dest_concls;
wenzelm [Thu, 04 Oct 2001 14:49:10 +0200] rev 11667
document setup;
wenzelm [Thu, 04 Oct 2001 11:29:46 +0200] rev 11666
added print_induct_rules;
wenzelm [Thu, 04 Oct 2001 11:29:25 +0200] rev 11665
tuned print operation;
wenzelm [Thu, 04 Oct 2001 11:29:02 +0200] rev 11664
tuned;
wenzelm [Thu, 04 Oct 2001 11:28:30 +0200] rev 11663
* moved induct/cases attributes to Pure, added 'print_induct_rules' command;
wenzelm [Thu, 04 Oct 2001 11:28:12 +0200] rev 11662
print_induct_rules;
wenzelm [Thu, 04 Oct 2001 11:22:10 +0200] rev 11661
updated;
berghofe [Thu, 04 Oct 2001 00:53:27 +0200] rev 11660
Fixed bug in decompose.
wenzelm [Wed, 03 Oct 2001 21:03:05 +0200] rev 11659
Tools/induct_attrib.ML now part of Pure;
wenzelm [Wed, 03 Oct 2001 21:01:53 +0200] rev 11658
Isar/induct_attrib.ML;
wenzelm [Wed, 03 Oct 2001 20:58:27 +0200] rev 11657
*** empty log message ***
wenzelm [Wed, 03 Oct 2001 20:55:31 +0200] rev 11656
moved HOL/Tools/induct_attrib.ML to Pure/Isar/induct_attrib.ML;
wenzelm [Wed, 03 Oct 2001 20:54:16 +0200] rev 11655
tuned parentheses in relational expressions;
wenzelm [Wed, 03 Oct 2001 20:54:05 +0200] rev 11654
moved linorder_cases to theory Ord;
wenzelm [Wed, 03 Oct 2001 20:53:02 +0200] rev 11653
linorder_cases supersedes linorder_less_split;
tuned parentheses in relational expressions;
paulson [Wed, 03 Oct 2001 11:45:24 +0200] rev 11652
eta-expansion required for SML/NJ
wenzelm [Tue, 02 Oct 2001 20:23:33 +0200] rev 11651
support non-oriented infix;
wenzelm [Mon, 01 Oct 2001 21:53:50 +0200] rev 11650
tuned;
wenzelm [Mon, 01 Oct 2001 15:46:35 +0200] rev 11649
tuned;
wenzelm [Mon, 01 Oct 2001 14:47:02 +0200] rev 11648
*** empty log message ***
wenzelm [Mon, 01 Oct 2001 14:44:00 +0200] rev 11647
initial setup for chapter on document preparation;
wenzelm [Mon, 01 Oct 2001 14:42:47 +0200] rev 11646
updated output;
streckem [Mon, 01 Oct 2001 13:39:17 +0200] rev 11645
- declared wf_java_prog as syntax (previously: definition)
- in wf_java_mdecl: added preconditions for 'This'
- rule LAss: precondition v ~=This
streckem [Mon, 01 Oct 2001 13:36:25 +0200] rev 11644
Removed some unfoldings of defs after declaring wf_java_prog as syntax
streckem [Mon, 01 Oct 2001 13:33:49 +0200] rev 11643
Added axiom e~=This to reflect strengthened precond. in rule LAss
streckem [Mon, 01 Oct 2001 13:32:11 +0200] rev 11642
Minor modifications
wenzelm [Mon, 01 Oct 2001 11:56:40 +0200] rev 11641
added Ordinals example;
berghofe [Sun, 30 Sep 2001 13:42:00 +0200] rev 11640
Tuned indentation of abstractions.
wenzelm [Fri, 28 Sep 2001 21:45:40 +0200] rev 11639
tuned;
wenzelm [Fri, 28 Sep 2001 21:45:11 +0200] rev 11638
inductive: no collective atts;
wenzelm [Fri, 28 Sep 2001 20:09:10 +0200] rev 11637
inductive: no collective atts;
wenzelm [Fri, 28 Sep 2001 20:08:28 +0200] rev 11636
oops;
wenzelm [Fri, 28 Sep 2001 20:08:05 +0200] rev 11635
tuned;
wenzelm [Fri, 28 Sep 2001 19:24:25 +0200] rev 11634
recdef (permissive);
inductive: no collective atts;
wenzelm [Fri, 28 Sep 2001 19:23:58 +0200] rev 11633
*** empty log message ***
wenzelm [Fri, 28 Sep 2001 19:23:35 +0200] rev 11632
prove: ``strict'' argument;
wenzelm [Fri, 28 Sep 2001 19:23:07 +0200] rev 11631
internal thm numbering with ":" instead of "_";
wenzelm [Fri, 28 Sep 2001 19:22:40 +0200] rev 11630
avoid handle _;
wenzelm [Fri, 28 Sep 2001 19:21:26 +0200] rev 11629
permissive option;
wenzelm [Fri, 28 Sep 2001 19:19:26 +0200] rev 11628
inductive: no collective atts;
wenzelm [Fri, 28 Sep 2001 19:18:46 +0200] rev 11627
updated;
wenzelm [Fri, 28 Sep 2001 19:17:01 +0200] rev 11626
recdef (permissive);
berghofe [Fri, 28 Sep 2001 18:55:37 +0200] rev 11625
Tuned section about parsing and printing proof terms.
berghofe [Fri, 28 Sep 2001 17:19:46 +0200] rev 11624
mksimps and mk_eq_True no longer raise THM exception.
berghofe [Fri, 28 Sep 2001 16:45:03 +0200] rev 11623
Added label for section on terms.
berghofe [Fri, 28 Sep 2001 16:44:27 +0200] rev 11622
Added documentation for proof terms.
berghofe [Fri, 28 Sep 2001 16:43:50 +0200] rev 11621
Added TYPE to Pure grammar.
berghofe [Fri, 28 Sep 2001 16:42:58 +0200] rev 11620
Added \ttlbrack and \ttrbrack.
berghofe [Fri, 28 Sep 2001 16:42:26 +0200] rev 11619
Added TPHOLs2000 paper about proof terms.
wenzelm [Fri, 28 Sep 2001 16:15:26 +0200] rev 11618
updated;
wenzelm [Fri, 28 Sep 2001 14:10:01 +0200] rev 11617
tuned;
wenzelm [Fri, 28 Sep 2001 14:04:14 +0200] rev 11616
tuned;
berghofe [Fri, 28 Sep 2001 11:08:53 +0200] rev 11615
- Exchanged % and %%.
- Fixed bug in shrink.
berghofe [Fri, 28 Sep 2001 11:07:40 +0200] rev 11614
- Tuned syntax
- proof_of_term: fixed problems with dummy patterns and typing information
berghofe [Fri, 28 Sep 2001 11:05:37 +0200] rev 11613
- Exchanged % and %%
- Renamed reconstruct_prf to reconstruct_proof
berghofe [Fri, 28 Sep 2001 11:04:44 +0200] rev 11612
Exchanged % and %%.
wenzelm [Thu, 27 Sep 2001 22:30:09 +0200] rev 11611
HOL: eliminated global items;
wenzelm [Thu, 27 Sep 2001 22:29:57 +0200] rev 11610
updated;
wenzelm [Thu, 27 Sep 2001 22:28:16 +0200] rev 11609
eliminated theories "equalities" and "mono" (made part of "Typedef",
which supercedes "subset");
wenzelm [Thu, 27 Sep 2001 22:26:00 +0200] rev 11608
renamed theory "subset" to "Typedef";
wenzelm [Thu, 27 Sep 2001 22:25:12 +0200] rev 11607
unsymbolize;
wenzelm [Thu, 27 Sep 2001 22:24:28 +0200] rev 11606
renamed "()" to Unity;
wenzelm [Thu, 27 Sep 2001 22:24:09 +0200] rev 11605
HOLogic.unit;
wenzelm [Thu, 27 Sep 2001 22:23:40 +0200] rev 11604
made unit type local;
wenzelm [Thu, 27 Sep 2001 22:23:20 +0200] rev 11603
tuned:
wenzelm [Thu, 27 Sep 2001 22:22:58 +0200] rev 11602
renamed "()" to Unity, made local;
wenzelm [Thu, 27 Sep 2001 22:22:08 +0200] rev 11601
added surjE;
wenzelm [Thu, 27 Sep 2001 18:56:39 +0200] rev 11600
prepared for Isabelle2001;
wenzelm [Thu, 27 Sep 2001 18:46:32 +0200] rev 11599
renamed real_of_nat_eq_cancel to real_of_nat_inject, and declared as iff rule;
wenzelm [Thu, 27 Sep 2001 18:45:40 +0200] rev 11598
updated;
wenzelm [Thu, 27 Sep 2001 18:45:23 +0200] rev 11597
renamed real_of_int_eq_iff to real_of_int_inject;
wenzelm [Thu, 27 Sep 2001 18:44:30 +0200] rev 11596
document setup;
wenzelm [Thu, 27 Sep 2001 18:44:12 +0200] rev 11595
new-style theory;
wenzelm [Thu, 27 Sep 2001 18:43:40 +0200] rev 11594
Square roots of primes are irrational;
wenzelm [Thu, 27 Sep 2001 18:43:17 +0200] rev 11593
AddXIs [dvdI]; AddXEs [dvdE];
added dvd_mult_div_cancel;
wenzelm [Thu, 27 Sep 2001 18:42:47 +0200] rev 11592
tuned;
wenzelm [Thu, 27 Sep 2001 16:43:46 +0200] rev 11591
tuned;
wenzelm [Thu, 27 Sep 2001 16:04:44 +0200] rev 11590
tuned;
wenzelm [Thu, 27 Sep 2001 16:04:25 +0200] rev 11589
AddXEs [UnI1, UnI2];
wenzelm [Thu, 27 Sep 2001 16:04:11 +0200] rev 11588
AddXEs [disjI1, disjI2];
wenzelm [Thu, 27 Sep 2001 15:42:30 +0200] rev 11587
ex/Hilbert_Classical.thy ex/document/root.tex;
wenzelm [Thu, 27 Sep 2001 15:42:08 +0200] rev 11586
tuned;
wenzelm [Thu, 27 Sep 2001 15:42:01 +0200] rev 11585
document setup;
wenzelm [Thu, 27 Sep 2001 15:41:48 +0200] rev 11584
derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm [Thu, 27 Sep 2001 14:35:40 +0200] rev 11583
obsolete;
wenzelm [Thu, 27 Sep 2001 12:25:09 +0200] rev 11582
updated;
wenzelm [Thu, 27 Sep 2001 12:24:40 +0200] rev 11581
-v option;
wenzelm [Thu, 27 Sep 2001 12:24:19 +0200] rev 11580
verbose option;
wenzelm [Thu, 27 Sep 2001 12:24:02 +0200] rev 11579
use_dir: verbose option;
wenzelm [Thu, 27 Sep 2001 12:23:23 +0200] rev 11578
removed option -d (now standard behaviour);
added option -q;
include notes;
wenzelm [Thu, 27 Sep 2001 12:22:45 +0200] rev 11577
option -v;
wenzelm [Wed, 26 Sep 2001 23:01:48 +0200] rev 11576
activate default ISABELLE_USEDIR_OPTIONS for precompiled distribution;
wenzelm [Wed, 26 Sep 2001 23:00:41 +0200] rev 11575
updated;
wenzelm [Wed, 26 Sep 2001 22:26:11 +0200] rev 11574
tuned order;
wenzelm [Wed, 26 Sep 2001 22:25:23 +0200] rev 11573
bold symbols;
wenzelm [Wed, 26 Sep 2001 22:24:55 +0200] rev 11572
tuned;