Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-240
+240
+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.
Locales and simple mathematical structures;
2001-11-06, by wenzelm
renamed Real/ex/Sqrt_Irrational.thy to Real/ex/Sqrt.thy;
2001-11-06, by wenzelm
extend_XXX: sane argument order ... -> syntax -> syntax;
2001-11-06, by wenzelm
local syntax: add_syntax, proper read/pretty functions;
2001-11-06, by wenzelm
locale_element/uses: string;
2001-11-06, by wenzelm
proper treatment of local syntax;
2001-11-06, by wenzelm
print_syntax: include local version;
2001-11-06, by wenzelm
added pretty_term', read_typ', read_typ_no_norm', read_def_terms'
2001-11-06, by wenzelm
export pretty_thm_aux;
2001-11-06, by wenzelm
tuned;
2001-11-06, by wenzelm
theorem(_i): locale atts;
2001-11-06, by wenzelm
group locale_element;
2001-11-06, by wenzelm
added add_locale(_i) and store_thm;
2001-11-06, by wenzelm
theorem(_i): locale atts;
2001-11-06, by wenzelm
added 'locale', 'print_locales', 'print_locale';
2001-11-06, by wenzelm
added print_locales, print_locale;
2001-11-06, by wenzelm
added "locale", "print_locale", "print_locales";
2001-11-06, by wenzelm
fixes: optional typ;
2001-11-05, by wenzelm
added pretty/print functions with context;
2001-11-05, by wenzelm
locale_element: optional typ;
2001-11-05, by wenzelm
pretty/print functions with context;
2001-11-05, by wenzelm
export add_tvarsT, add_tvars, add_vars, add_frees (would actually
2001-11-05, by wenzelm
Method.trace ctxt;
2001-11-05, by wenzelm
tuned;
2001-11-05, by wenzelm
new Sqrt example
2001-11-05, by paulson
tuned comment;
2001-11-04, by wenzelm
simplified Proof.init_state:
2001-11-04, by wenzelm
added get_thms_with_closure;
2001-11-04, by wenzelm
added locale_element;
2001-11-04, by wenzelm
locale elements;
2001-11-04, by wenzelm
theorem(_i): locale elements;
2001-11-04, by wenzelm
locale syntax;
2001-11-04, by wenzelm
IsarThy.theorem_i (None, []);
2001-11-04, by wenzelm
updated;
2001-11-04, by wenzelm
Fixed bug in function add_npvars.
2001-11-03, by berghofe
updated;
2001-11-03, by wenzelm
tuned;
2001-11-03, by wenzelm
proper use of bind_thm(s);
2001-11-03, by wenzelm
adapted to new-style theories;
2001-11-03, by wenzelm
GPLed;
2001-11-03, by wenzelm
converted theory Dnat;
2001-11-03, by wenzelm
* 'domain' package adapted to new-style theories, e.g. see
2001-11-03, by wenzelm
document setup;
2001-11-03, by wenzelm
replaced Undef by UU;
2001-11-03, by wenzelm
ax_flat;
2001-11-03, by wenzelm
GPLed;
2001-11-03, by wenzelm
tuned;
2001-11-03, by wenzelm
replaced Undef by UU;
2001-11-03, by wenzelm
converted theory Lift;
2001-11-03, by wenzelm
rep_datatype lift;
2001-11-03, by wenzelm
moved into Main;
2001-11-03, by wenzelm
moved String into Main;
2001-11-03, by wenzelm
tuned;
2001-11-03, by wenzelm
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
iff: always rotate prems;
2001-10-23, by wenzelm
apply(simp add: three_def numerals) (* FIXME !? *);
2001-10-23, by wenzelm
unset DISPLAY (again);
2001-10-23, by wenzelm
* Pure: removed obsolete 'exported' attribute;
2001-10-23, by wenzelm
*** empty log message ***
2001-10-22, by wenzelm
moved object_logic.ML to Isar/object_logic.ML;
2001-10-22, by wenzelm
moved locale.ML to Isar/locale.ML;
2001-10-22, by wenzelm
moved goal related stuff to goals.ML;
2001-10-22, by wenzelm
Display.current_goals_markers;
2001-10-22, by wenzelm
tuned;
2001-10-22, by wenzelm
moved prove_goalw_cterm to goals.ML;
2001-10-22, by wenzelm
moved local defs to proof.ML (for locales);
2001-10-22, by wenzelm
improved source arrangement of obtain;
2001-10-22, by wenzelm
rearrange sources for locales;
2001-10-22, by wenzelm
Display.print_current_goals_fn;
2001-10-22, by wenzelm
Display.print_goals;
2001-10-22, by wenzelm
Display.pretty_thms;
2001-10-22, by wenzelm
qualified names;
2001-10-22, by wenzelm
make this module appeat late in Pure;
2001-10-22, by wenzelm
print_goals stuff is back (from locale.ML);
2001-10-22, by wenzelm
reorganize sources to accomodate locales;
2001-10-22, by wenzelm
corollary;
2001-10-22, by wenzelm
quick_and_dirty_prove_goalw_cterm;
2001-10-22, by wenzelm
javac -depend;
2001-10-22, by wenzelm
-D generated;
2001-10-22, by wenzelm
Added "clean" target.
2001-10-22, by berghofe
Fixed problem with batch mode layout, which caused an AWT exception when
2001-10-22, by berghofe
initBrowser now has additional noAWT argument.
2001-10-22, by berghofe
Constructor no longer takes font as an argument.
2001-10-22, by berghofe
Moved font settings from TreeNode to TreeBrowser.
2001-10-22, by berghofe
Moved font settings from Vertex to GraphView.
2001-10-22, by berghofe
deleted the redundant first argument of adjust(a,b)
2001-10-22, by paulson
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
2001-10-22, by paulson
New simproc, needed to cope with combinations of (abstract) 0, (abstract) 1,
2001-10-22, by paulson
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
2001-10-22, by paulson
keep DISPLAY;
2001-10-22, by wenzelm
updated;
2001-10-21, by wenzelm
renamed to Typedefs.thy to avoid conflict with main HOL version;
2001-10-21, by wenzelm
* proper spacing of consecutive markup elements, especially text
2001-10-21, by wenzelm
\newif\ifisamarkup controls spacing of isabeginpar;
2001-10-21, by wenzelm
improved spacing;
2001-10-21, by wenzelm
maintain Latex.flag_markup;
2001-10-21, by wenzelm
flag_markup;
2001-10-21, by wenzelm
Types/document/Typedefs;
2001-10-21, by wenzelm
renamed Typedef.thy to Typedefs.thy (former already present in main HOL);
2001-10-21, by wenzelm
got rid of separate root.tex;
2001-10-20, by wenzelm
graceful interpretation of -i/-d/-D options;
2001-10-20, by wenzelm
include document graph;
2001-10-20, by wenzelm
document graph option;
2001-10-20, by wenzelm
conditional: bool -> (unit -> unit) -> unit;
2001-10-20, by wenzelm
added TextIO.stdErr;
2001-10-20, by wenzelm
include document graph;
2001-10-20, by wenzelm
document graphs for several sessions;
2001-10-20, by wenzelm
tuned;
2001-10-20, by wenzelm
calculational rules moved from FOL to IFOL;
2001-10-20, by wenzelm
option -g for document graph;
2001-10-20, by wenzelm
option -q also excludes -v true in generated stuff;
2001-10-20, by wenzelm
dvips -q;
2001-10-20, by wenzelm
removed -v option (handled by isabelle process);
2001-10-20, by wenzelm
-o pdf: produce *both* eps and pdf;
2001-10-20, by wenzelm
* greatly simplified document preparation setup, including more
2001-10-20, by wenzelm
got rid of ML proof scripts;
2001-10-19, by wenzelm
induct_method.ML -- proof by cases and induction on sets and types (Isar);
2001-10-19, by wenzelm
latex output: bold lambda;
2001-10-19, by wenzelm
got rid of ML proof scripts for Product_Type;
2001-10-19, by wenzelm
got rid of Provers/split_paired_all.ML;
2001-10-19, by wenzelm
improved default dependencies;
2001-10-19, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip