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.
even more theories from Jacques
2001-11-16, by paulson
finish_global: Drule.strip_shyps_warning (just for warning);
2001-11-16, by wenzelm
ext_tsig_classes: rebuild_tsig!!!!!
2001-11-16, by wenzelm
local_standard: plain strip_shyps instead of strip_shyps_warning;
2001-11-16, by wenzelm
last-minute tidying
2001-11-16, by paulson
updated;
2001-11-15, by wenzelm
GPLed;
2001-11-15, by wenzelm
write_keywords: string argument (logic name);
2001-11-15, by wenzelm
isatool unsymbolize;
2001-11-15, by wenzelm
Modified to make the files build with the new changes in ZF
2001-11-15, by ehmety
depends on Epsilon!
2001-11-15, by wenzelm
fix_frees: rev;
2001-11-15, by wenzelm
prove: raise ERROR_MESSAGE;
2001-11-15, by wenzelm
updated;
2001-11-15, by wenzelm
* ZF: new-style theory commands '(co)inductive', '(co)datatype',
2001-11-15, by wenzelm
type_solver_tac: use TCSET' to refer to context of goal state (does
2001-11-15, by wenzelm
setup DatatypeTactics.setup;
2001-11-15, by wenzelm
added Induct/Binary_Trees.thy, Induct/Tree_Forest (converted from
2001-11-15, by wenzelm
no handle ERROR;
2001-11-15, by wenzelm
fixed;
2001-11-15, by wenzelm
Isar version of 'rep_datatype';
2001-11-15, by wenzelm
avoid handle _;
2001-11-15, by wenzelm
added TCSET(') tacticals;
2001-11-15, by wenzelm
added Term and Tree_Forest (from converted ZF/ex);
2001-11-15, by wenzelm
TF and Term moved to ZF/Induct;
2001-11-15, by wenzelm
miniscoping of UN and INT
2001-11-15, by paulson
Added new entry
2001-11-15, by ehmety
New files
2001-11-15, by ehmety
new theories from Jacques Fleuriot
2001-11-15, by paulson
*** empty log message ***
2001-11-15, by ehmety
converted datatype examples moved from ZF/ex to ZF/Induct;
2001-11-14, by wenzelm
document setup;
2001-11-14, by wenzelm
removed BT, Data, Enum (see ZF/Induct);
2001-11-14, by wenzelm
case_names;
2001-11-14, by wenzelm
added Datatypes, Binary_Trees (from ZF/ex);
2001-11-14, by wenzelm
Isar attribute and method setup;
2001-11-14, by wenzelm
fix path prefix;
2001-11-14, by wenzelm
use proper intr_names (for required case_names);
2001-11-14, by wenzelm
added Induct/Binary_Trees.thy, Induct/Datatypes.thy;
2001-11-14, by wenzelm
tuned;
2001-11-14, by wenzelm
updated;
2001-11-14, by wenzelm
adapted primrec/datatype to Isar;
2001-11-14, by wenzelm
tuned;
2001-11-14, by wenzelm
store original simps for codegen;
2001-11-14, by wenzelm
inductive: removed con_defs;
2001-11-14, by wenzelm
updated;
2001-11-14, by wenzelm
updated;
2001-11-13, by wenzelm
* ZF: new-style theory commands 'inductive', 'inductive_cases', and
2001-11-13, by wenzelm
ZF specific keywords;
2001-11-13, by wenzelm
rearranged inductive package for Isar;
2001-11-13, by wenzelm
Generic inductive cases facility for (co)inductive definitions.
2001-11-13, by wenzelm
converted;
2001-11-13, by wenzelm
tuned;
2001-11-13, by wenzelm
tuned inductions;
2001-11-13, by wenzelm
prove: Envir.beta_norm;
2001-11-13, by wenzelm
new SList theory from Bu Wolff
2001-11-13, by paulson
induct: rule_versions produces localized variants;
2001-11-12, by wenzelm
empty rule_context for multiple goals;
2001-11-12, by wenzelm
added empty;
2001-11-12, by wenzelm
mutual rules declared as ``consumes 0'';
2001-11-12, by wenzelm
induct_atomize: include atomize_conj (for mutual induction);
2001-11-12, by wenzelm
Isar: 'induct' proper support for mutual induction involving
2001-11-12, by wenzelm
proper handling of mutual rules (esp. for sets);
2001-11-12, by wenzelm
lemmas induct_atomize = atomize_conj ...;
2001-11-12, by wenzelm
val local_imp_def = thm "induct_implies_def";
2001-11-12, by wenzelm
ZF/Induct,UNITY
2001-11-12, by paulson
Tidying necessitated by new simprules in equalities.ML
2001-11-12, by paulson
conditional miniscoping equalities now made unconditional
2001-11-12, by paulson
new-style numerals without leading #, along with generic 0 and 1
2001-11-12, by paulson
congc now returns None if congruence rule has no effect.
2001-11-12, by berghofe
Renamed some bound variables due to changes in simplifier.
2001-11-12, by berghofe
Fixed proof depending on strange behaviour of rename_bvs.
2001-11-12, by berghofe
Renamed some bound variables due to changes in simplifier.
2001-11-12, by berghofe
present multi_result;
2001-11-11, by wenzelm
added meta_conjunction_tr';
2001-11-11, by wenzelm
pure_syntax_output: "_meta_conjunction";
2001-11-11, by wenzelm
adapted to multiple results;
2001-11-11, by wenzelm
adapted auto_bind_goal, auto_bind_facts;
2001-11-11, by wenzelm
added multi_theorem(_i);
2001-11-11, by wenzelm
Proof.have_i: multiple statements;
2001-11-11, by wenzelm
added RAW_METHOD, RAW_METHOD_CASES;
2001-11-11, by wenzelm
added add_thmss;
2001-11-11, by wenzelm
"theorem" etc.: multiple statements;
2001-11-11, by wenzelm
theorem, have, show etc: multiple statements;
2001-11-11, by wenzelm
facts: multiple args;
2001-11-11, by wenzelm
added conjunction_tac;
2001-11-11, by wenzelm
renamed open_smart_store_thms to smart_store_thms_open;
2001-11-11, by wenzelm
added mk_conjunction;
2001-11-11, by wenzelm
added unflat;
2001-11-11, by wenzelm
added conj_elim_precise, conj_intr_thm;
2001-11-11, by wenzelm
use Tactic.prove;
2001-11-10, by wenzelm
tuned;
2001-11-09, by wenzelm
support co/inductive definitions in new-style theories;
2001-11-09, by wenzelm
adapted to add_inductive_x;
2001-11-09, by wenzelm
syntactic declaration of external *and* internal versions of fixes;
2001-11-09, by wenzelm
fixed print_records;
2001-11-09, by wenzelm
tuned;
2001-11-09, by wenzelm
theorems case_split = case_split_thm [case_names True False, cases type: o];
2001-11-09, by wenzelm
Theorems symmetric, reflexive and transitive are now stored with "open"
2001-11-09, by berghofe
Commands prf and full_prf can now also be used to display proof term
2001-11-09, by berghofe
eliminated old "symbols" syntax, use "xsymbols" instead;
2001-11-09, by wenzelm
theory data: finish method;
2001-11-09, by wenzelm
indexvar_ast_tr (for \<index> placeholder);
2001-11-09, by wenzelm
removed pure_sym_syntax;
2001-11-09, by wenzelm
File.use;
2001-11-09, by wenzelm
added impose_hyps_tac;
2001-11-09, by wenzelm
proper close_locale;
2001-11-09, by wenzelm
no longer support "isabelle_font" or "symbols";
2001-11-09, by wenzelm
got rid of obsolete input filtering;
2001-11-09, by wenzelm
back to normal;
2001-11-09, by wenzelm
eliminated old "symbols" syntax, use "xsymbols" instead;
2001-11-09, by wenzelm
updated;
2001-11-09, by wenzelm
got rid of obsolete input filtering and isabelle font encoding;
2001-11-09, by wenzelm
got rid of obsolete input filtering;
2001-11-09, by wenzelm
eliminated old "symbols" syntax, use "xsymbols" instead;
2001-11-09, by wenzelm
theory data: finish method;
2001-11-08, by wenzelm
removed needs_filtered_use;
2001-11-08, by wenzelm
\newcommand{\isasymindex}{\isamath{\i}};
2001-11-08, by wenzelm
* Isar/Pure: emulation of instantiation tactics (rule_tac, cut_tac,
2001-11-08, by wenzelm
tuned;
2001-11-08, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip