Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-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.
installation of cancellation simprocs for the integers
2000-08-10, by paulson
X-Symbol mode -- look in canonical place;
2000-08-10, by wenzelm
fixed spelling;
2000-08-09, by wenzelm
added Bauer-Wenzel:2000:HB;
2000-08-09, by wenzelm
thms closure;
2000-08-09, by wenzelm
res_inst: include non-inst versions with multiple thms;
2000-08-09, by wenzelm
added get_thms_closure, single_thm;
2000-08-09, by wenzelm
fixed classification of rules in atts and modifiers (final!?);
2000-08-09, by wenzelm
fixed mk_cases_i: TRYALL InductMethod.simp_case_tac;
2000-08-09, by wenzelm
thms "atomize";
2000-08-09, by wenzelm
tuned;
2000-08-09, by bauerg
tuned
2000-08-09, by kleing
token translation: enclose "\\mbox{" "}";
2000-08-08, by wenzelm
added Example
2000-08-08, by oheimb
moved Hoare_example to Examples; other minor improvements
2000-08-08, by oheimb
Deleted unneeded proof; simplified proof of app_last.
2000-08-08, by berghofe
added forall_elim_vars_safe, norm_hhf_eq;
2000-08-08, by wenzelm
norm_hhf results;
2000-08-08, by wenzelm
prf_heading kind;
2000-08-08, by wenzelm
MicroJava structure changed
2000-08-07, by kleing
Invoke instruction gets fully qualified method name (class+name+sig) as
2000-08-07, by kleing
BV and LBV specified in terms of app and step functions
2000-08-07, by kleing
instantiated Cancel_Numerals for "nat" in ZF
2000-08-07, by paulson
more cterm operations: mk_implies, list_implies
2000-08-07, by paulson
prove_conv gets an extra argument, so the ZF instantiation can use hyps
2000-08-07, by paulson
tidied
2000-08-07, by paulson
added a dummy "thm list" argument to prove_conv for the new interface to
2000-08-07, by paulson
new abstract syntax operations, used in ZF
2000-08-07, by paulson
ZF arith
2000-08-07, by paulson
*** empty log message ***
2000-08-06, by nipkow
dummy_patterns moved to term.ML;
2000-08-04, by wenzelm
added goal_args(');
2000-08-04, by wenzelm
added int;
2000-08-04, by wenzelm
axioms: Term.no_dummy_patterns;
2000-08-04, by wenzelm
added dummy_patternN, no_dummy_patterns, replace_dummy_patterns;
2000-08-04, by wenzelm
added rename_params_tac;
2000-08-04, by wenzelm
dummy_pattern moved to term.ML;
2000-08-04, by wenzelm
Term.no_dummy_patterns;
2000-08-04, by wenzelm
added rev_eq_reflection;
2000-08-04, by wenzelm
val rev_eq_reflection = def_imp_eq;
2000-08-04, by wenzelm
val atomize = thms "atomize";
2000-08-04, by wenzelm
lemmas atomize = all_eq imp_eq;
2000-08-04, by wenzelm
rev_eq_reflection = meta_eq_to_obj_eq;
2000-08-04, by wenzelm
removed stac (now exported by HypsubstFun);
2000-08-04, by wenzelm
setup hypsubst_setup;
2000-08-04, by wenzelm
lemmas atomize = all_eq imp_eq;
2000-08-04, by wenzelm
added rev_eq_reflection;
2000-08-04, by wenzelm
subgoals_tac: fixed spelling;
2000-08-04, by wenzelm
invoke isatool make in any dir containing an IsaMakefile;
2000-08-04, by wenzelm
updated;
2000-08-04, by wenzelm
targets for images, test, all;
2000-08-04, by wenzelm
updated;
2000-08-04, by wenzelm
tuned;
2000-08-04, by wenzelm
tuned version by Stephan Merz (unbatchified etc.);
2000-08-03, by wenzelm
tuned TLA;
2000-08-03, by wenzelm
added setmp_verbose;
2000-08-03, by wenzelm
tuned;
2000-08-03, by wenzelm
unknown_theory/proof/context;
2000-08-03, by wenzelm
added unknown_theory/proof/context;
2000-08-03, by wenzelm
new theorem neq_commute
2000-08-03, by paulson
new files Integ/IntPower.{thy.ML}; tidied
2000-08-03, by paulson
introduction of integer exponentiation
2000-08-03, by paulson
Chinese Remainder Theorem, Wilsons Theorem, etc., by T M Masmussen
2000-08-03, by paulson
GPLed;
2000-08-03, by wenzelm
export get_local_clasimpset, clasimp_modifiers;
2000-08-03, by wenzelm
improved output of space symbol;
2000-08-03, by wenzelm
typ_no_norm;
2000-08-03, by wenzelm
tuned;
2000-08-03, by wenzelm
adapted deriv;
2000-08-02, by wenzelm
derivations: maintain oracle flag;
2000-08-02, by wenzelm
use oracle flag from derivation;
2000-08-02, by wenzelm
rep_thm: 'der' field has additional bool for oracles;
2000-08-02, by wenzelm
minor corrections
2000-08-02, by oheimb
isa: do not touch_all_thys on startup;
2000-08-02, by wenzelm
coercion "intify" to remove type constraints from integer algebraic laws
2000-08-02, by paulson
tidying and speeding up proofs
2000-08-02, by paulson
*** empty log message ***
2000-08-02, by nipkow
*** empty log message ***
2000-08-02, by nipkow
used natify with div and mod; also put in the divide-by-zero trick
2000-08-01, by paulson
natify, a coercion to reduce the number of type constraints in arithmetic
2000-08-01, by paulson
tuned msg;
2000-08-01, by wenzelm
* blast(_tac) now handles actual object-logic rules as assumptions;
2000-08-01, by wenzelm
added all_eq, imp_eq (for blast);
2000-08-01, by wenzelm
improved comments;
2000-08-01, by wenzelm
handle actual object-logic rules by atomizing the goal;
2000-08-01, by wenzelm
added atomize_goal / atomize_tac;
2000-08-01, by wenzelm
(un)fold: CHANGED;
2000-08-01, by wenzelm
added has_meta_prems;
2000-08-01, by wenzelm
tuned;
2000-08-01, by wenzelm
tuned;
2000-07-31, by wenzelm
updated 'obtain';
2000-07-31, by wenzelm
Removed Quot
2000-07-31, by nipkow
Never used and not relevant.
2000-07-31, by nipkow
obtain;
2000-07-30, by wenzelm
added split_bind_asm, bind_splits;
2000-07-30, by wenzelm
adapted obtain;
2000-07-30, by wenzelm
removed equalityCE;
2000-07-30, by wenzelm
added atomic_Trueprop;
2000-07-30, by wenzelm
updated ObtainFun;
2000-07-30, by wenzelm
'def': no constraint on variable;
2000-07-30, by wenzelm
exporter setup for context elements;
2000-07-30, by wenzelm
export RANGE, hard_asm_tac, soft_asm_tac;
2000-07-30, by wenzelm
turned into plain context element;
2000-07-30, by wenzelm
local_def(_i): no constraint on var;
2000-07-30, by wenzelm
local_def(_i): no constraint on var;
2000-07-30, by wenzelm
def: no constraint on var;
2000-07-30, by wenzelm
added is_judgment;
2000-07-30, by wenzelm
ObtainFun (generalized existence reasoning);
2000-07-30, by wenzelm
ThmDeps.enable;
2000-07-30, by wenzelm
added sign_of_cterm;
2000-07-30, by wenzelm
Logic.goal_const;
2000-07-30, by wenzelm
replaced "Sessions" by "Root";
2000-07-28, by wenzelm
apply. -> by
2000-07-28, by nipkow
* HOL/While
2000-07-28, by nipkow
added theory While;
2000-07-27, by wenzelm
export has_internal;
2000-07-27, by wenzelm
added thm_deps;
2000-07-27, by wenzelm
added enter_forward_proof;
2000-07-27, by wenzelm
export write_graph;
2000-07-27, by wenzelm
begin_theory: store *copy* of initial theory;
2000-07-27, by wenzelm
less
more
|
(0)
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip