Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
HOLCF: proper rep_datatype lift (see theory Lift); use plain induct_tac
2001-11-03, by wenzelm
declare transitive;
2001-11-02, by wenzelm
theory Calculation move to Set;
2001-11-02, by wenzelm
transitive declared in Pure;
2001-11-02, by wenzelm
Numerals and simprocs for types real and hypreal. The abstract
2001-11-02, by paulson
Goals.add_locale;
2001-11-01, by wenzelm
fix_frees;
2001-11-01, by wenzelm
theorem: locale argument;
2001-11-01, by wenzelm
beginnings of new locales (not yet functional);
2001-11-01, by wenzelm
Goals.setup;
2001-11-01, by wenzelm
parking code for old-style locales here;
2001-11-01, by wenzelm
tuned notation (degree instead of dollar);
2001-10-31, by wenzelm
theorem(_i): locale argument;
2001-10-31, by wenzelm
Proof.init_state thy None;
2001-10-31, by wenzelm
simplified export;
2001-10-31, by wenzelm
'atomize': CHANGED_PROP;
2001-10-31, by wenzelm
global statements: locale argument;
2001-10-31, by wenzelm
added local_standard;
2001-10-31, by wenzelm
IsarThy.theorem_i: no locale;
2001-10-31, by wenzelm
removed obsolete (rule equal_intr_rule);
2001-10-31, by wenzelm
Additional rules for simplifying inside "Goal"
2001-10-31, by berghofe
- Tuned add_cnstrt
2001-10-31, by berghofe
Removed name_thm from finish_global.
2001-10-31, by berghofe
Tuned function thm_proof.
2001-10-31, by berghofe
- enter_thmx -> enter_thms
2001-10-31, by berghofe
norm_hhf_eq is now stored using open_store_standard_thm.
2001-10-31, by berghofe
induct: internalize ``missing'' consumes-facts from goal state
2001-10-31, by wenzelm
- 'induct' may now use elim-style induction rules without chaining
2001-10-31, by wenzelm
(induct set: ...);
2001-10-31, by wenzelm
put_consumes: really overwrite existing tag;
2001-10-31, by wenzelm
finish_global: Tactic.norm_hhf;
2001-10-31, by wenzelm
use HOL.induct_XXX;
2001-10-31, by wenzelm
use induct_rulify2;
2001-10-31, by wenzelm
renamed inductive_XXX to induct_XXX;
2001-10-31, by wenzelm
induct_impliesI;
2001-10-31, by wenzelm
tuned induct proofs;
2001-10-30, by wenzelm
- 'induct' method now derives symbolic cases from the *rulified* rule
2001-10-30, by wenzelm
tuned;
2001-10-30, by wenzelm
induct: cases are extracted from rulified rule;
2001-10-30, by wenzelm
removed obsolete make_raw;
2001-10-30, by wenzelm
lemma Least_mono moved from Typedef.thy to Set.thy;
2001-10-30, by wenzelm
tuned;
2001-10-29, by wenzelm
removed option -depend (not available everywhere?);
2001-10-29, by wenzelm
converted theory "Set";
2001-10-28, by wenzelm
fixed string_of_mixfix;
2001-10-28, by wenzelm
tuned declaration of rules;
2001-10-28, by wenzelm
equal_intr_rule already declared in Pure;
2001-10-28, by wenzelm
rules for meta-level conjunction;
2001-10-28, by wenzelm
tuned prove;
2001-10-28, by wenzelm
tuned;
2001-10-27, by wenzelm
added prove;
2001-10-27, by wenzelm
declare equal_intr_rule as intro;
2001-10-27, by wenzelm
tuned prove;
2001-10-27, by wenzelm
removed obsolete goal_subclass, goal_arity;
2001-10-27, by wenzelm
use Tactic.prove;
2001-10-27, by wenzelm
use Tactic.prove;
2001-10-27, by wenzelm
tuned;
2001-10-27, by wenzelm
* Pure/axclass: removed obsolete ML interface goal_subclass/goal_arity;
2001-10-27, by wenzelm
updated;
2001-10-27, by wenzelm
impose hyps on initial goal configuration (prevents res_inst_tac problems);
2001-10-27, by wenzelm
added "atomize" method;
2001-10-27, by wenzelm
prove: primitive goal interface for internal use;
2001-10-27, by wenzelm
added impose_hyps;
2001-10-27, by wenzelm
exclude field_simps from user-level "simps";
2001-10-27, by wenzelm
Isar: fixed rep_datatype args;
2001-10-27, by wenzelm
hardwire qualified const names;
2001-10-27, by wenzelm
removed "more" class;
2001-10-27, by wenzelm
moved product cases/induct to theory Datatype;
2001-10-27, by wenzelm
made new-style theory;
2001-10-27, by wenzelm
atomize_conj;
2001-10-26, by wenzelm
* Pure: method 'atomize' presents local goal premises as object-level
2001-10-26, by wenzelm
Fixed several bugs concerning arbitrarily branching datatypes.
2001-10-26, by berghofe
Eliminated occurrence of rule_format.
2001-10-26, by berghofe
tuned;
2001-10-26, by wenzelm
need at least 3 latex runs to get toc right!
2001-10-26, by wenzelm
tuned;
2001-10-26, by wenzelm
tuned;
2001-10-26, by wenzelm
Rrightarrow;
2001-10-26, by wenzelm
tuned notation;
2001-10-26, by wenzelm
tuned notation;
2001-10-26, by wenzelm
accomodate some recent changes of record package;
2001-10-25, by wenzelm
updated;
2001-10-25, by wenzelm
removed "more" sort;
2001-10-25, by wenzelm
updated records;
2001-10-25, by wenzelm
'simplified' att: args;
2001-10-25, by wenzelm
* HOL/record:
2001-10-25, by wenzelm
* Provers: 'simplified' attribute may refer to explicit rules instead
2001-10-25, by wenzelm
Replaced main proof by proper Isar script.
2001-10-25, by berghofe
derived operations are now: make, extend, truncate (cf. derived_defs);
2001-10-25, by wenzelm
tuned;
2001-10-25, by wenzelm
check_goal: setmp proofs 0;
2001-10-25, by wenzelm
added windowlistener (can now close the frame by window controls)
2001-10-25, by kleing
* HOL/record:
2001-10-25, by wenzelm
innermost_params;
2001-10-25, by wenzelm
(simp add: point.make_def);
2001-10-25, by wenzelm
provodes induct/cases for use with corresponding Isar methods;
2001-10-25, by wenzelm
further 1.73 changes: added fix_direct, simplified assume interface;
2001-10-24, by wenzelm
added read_prop_schematic;
2001-10-24, by wenzelm
simplified ProofContext.assume interface;
2001-10-24, by wenzelm
moved lambda to Pure/term.ML;
2001-10-24, by wenzelm
added lambda;
2001-10-24, by wenzelm
* clasimp: ``iff'' declarations now handle conditional rules as well;
2001-10-24, by wenzelm
added string_of_mixfix;
2001-10-24, by wenzelm
print_depth 8 from the very beginning;
2001-10-24, by wenzelm
added export_assume, export_presume, export_def (from proof.ML);
2001-10-23, by wenzelm
moved RANGE to tctical.ML;
2001-10-23, by wenzelm
added RANGE (from Isar/proof.ML);
2001-10-23, by wenzelm
print fixed names as plain strings;
2001-10-23, by wenzelm
eliminated old numerals;
2001-10-23, by wenzelm
use generic 1 instead of Numeral1;
2001-10-23, by wenzelm
eliminated Numeral0;
2001-10-23, by wenzelm
build option enables most basic browser info (for proper recording of session);
2001-10-23, by wenzelm
build option;
2001-10-23, by wenzelm
tuned;
2001-10-23, by wenzelm
eliminated old numerals;
2001-10-23, by wenzelm
pass build mode to process;
2001-10-23, by wenzelm
removed export_thm;
2001-10-23, by wenzelm
trace_rules: only non-empty;
2001-10-23, by wenzelm
removed obsolete "exported" att;
2001-10-23, by wenzelm
replace_dummy_patterns: lift over bounds;
2001-10-23, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip