berghofe [Wed, 11 Jul 2007 11:43:31 +0200] rev 23764
New wrapper for defining inductive sets with new inductive
predicate package.
berghofe [Wed, 11 Jul 2007 11:41:30 +0200] rev 23763
Old (co)inductive command is now replaced by (co)inductive_set.
berghofe [Wed, 11 Jul 2007 11:39:59 +0200] rev 23762
Reorganization due to introduction of inductive_set wrapper.
berghofe [Wed, 11 Jul 2007 11:38:25 +0200] rev 23761
Improved code generator for Collect.
berghofe [Wed, 11 Jul 2007 11:36:06 +0200] rev 23760
Renamed inductive2 to inductive.
aspinall [Wed, 11 Jul 2007 11:35:17 +0200] rev 23759
Fix nested PGIP messages. Update for schema simplifications.
berghofe [Wed, 11 Jul 2007 11:34:38 +0200] rev 23758
Moved unify_consts to PrimrecPackage.
berghofe [Wed, 11 Jul 2007 11:32:02 +0200] rev 23757
- Renamed inductive2 to inductive
- Renamed some theorems about transitive closure for predicates
berghofe [Wed, 11 Jul 2007 11:29:44 +0200] rev 23756
Adapted to changes in Predicate theory.
berghofe [Wed, 11 Jul 2007 11:28:13 +0200] rev 23755
Adapted to new inductive definition package.
berghofe [Wed, 11 Jul 2007 11:27:46 +0200] rev 23754
Renamed accessible part for predicates to accp.
aspinall [Wed, 11 Jul 2007 11:25:24 +0200] rev 23753
Track schema changes: merge messagecategory with area attributes
berghofe [Wed, 11 Jul 2007 11:25:21 +0200] rev 23752
bot is now a constant.
berghofe [Wed, 11 Jul 2007 11:24:36 +0200] rev 23751
Restored set notation.
berghofe [Wed, 11 Jul 2007 11:23:24 +0200] rev 23750
- Renamed inductive2 to inductive
- Renamed some theorems about transitive closure for predicates
aspinall [Wed, 11 Jul 2007 11:22:02 +0200] rev 23749
Track schema changes: remove cleardisplay, proofstate messages. Simplify attributes on cleardisplay, normalresponse.
aspinall [Wed, 11 Jul 2007 11:21:10 +0200] rev 23748
Track schema changes: add area attribute to pgml packet. Also add quoted Raw element [hack for Isabelle bottom-up XML production]
berghofe [Wed, 11 Jul 2007 11:16:34 +0200] rev 23747
Renamed inductive2 to inductive.
berghofe [Wed, 11 Jul 2007 11:14:51 +0200] rev 23746
Adapted to new inductive definition package.
berghofe [Wed, 11 Jul 2007 11:13:08 +0200] rev 23745
New operations on tuples with specific arities.
berghofe [Wed, 11 Jul 2007 11:11:39 +0200] rev 23744
Adapted to changes in infrastructure for converting between
sets and predicates.
berghofe [Wed, 11 Jul 2007 11:10:37 +0200] rev 23743
rtrancl and trancl are now defined using inductive_set.
berghofe [Wed, 11 Jul 2007 11:09:15 +0200] rev 23742
Removed wf_implies_wfP and wfP_implies_wf from list of hints again.
berghofe [Wed, 11 Jul 2007 11:07:57 +0200] rev 23741
- Moved infrastructure for converting between sets and predicates
to Tools/inductive_set_package.ML
- Adapted conversion rules to new format (now use standard op :
and Collect operators rather than Collect2 and member(2))
- Removed bounded quantifiers for predicates
berghofe [Wed, 11 Jul 2007 11:04:39 +0200] rev 23740
Adapted to new package for inductive sets.
berghofe [Wed, 11 Jul 2007 11:03:11 +0200] rev 23739
Inserted definition of in_rel again (since member2 was removed).
berghofe [Wed, 11 Jul 2007 11:02:07 +0200] rev 23738
Added ML bindings for sup_fun_eq and sup_bool_eq.
berghofe [Wed, 11 Jul 2007 11:01:24 +0200] rev 23737
top and bot are now constants.
berghofe [Wed, 11 Jul 2007 11:00:46 +0200] rev 23736
Renamed inductive2 to inductive.
berghofe [Wed, 11 Jul 2007 11:00:09 +0200] rev 23735
acc is now defined using inductive_set.
berghofe [Wed, 11 Jul 2007 10:59:23 +0200] rev 23734
Added new package for inductive sets.
berghofe [Wed, 11 Jul 2007 10:53:39 +0200] rev 23733
Adapted to new inductive definition package.
berghofe [Wed, 11 Jul 2007 10:52:20 +0200] rev 23732
Adapted to changes in inductive definition package.
wenzelm [Wed, 11 Jul 2007 00:46:48 +0200] rev 23731
tuned comment markup;
wenzelm [Wed, 11 Jul 2007 00:29:52 +0200] rev 23730
treat OuterLex.Error;
wenzelm [Wed, 11 Jul 2007 00:29:51 +0200] rev 23729
separated Malformed (symbolic char) from Error (bad input);
unparse: Output.escape_malformed;
name_of: use unparse;
wenzelm [Wed, 11 Jul 2007 00:29:50 +0200] rev 23728
Output.escape_malformed;
wenzelm [Wed, 11 Jul 2007 00:29:49 +0200] rev 23727
added escape_malformed (failsafe);
wenzelm [Tue, 10 Jul 2007 23:29:53 +0200] rev 23726
Basic editing of theory sources.
wenzelm [Tue, 10 Jul 2007 23:29:52 +0200] rev 23725
tuned;
wenzelm [Tue, 10 Jul 2007 23:29:51 +0200] rev 23724
export html_mode, begin_document, end_document;
wenzelm [Tue, 10 Jul 2007 23:29:49 +0200] rev 23723
renamed XML.Rawtext to XML.Output;
wenzelm [Tue, 10 Jul 2007 23:29:47 +0200] rev 23722
export get_lexicons;
wenzelm [Tue, 10 Jul 2007 23:29:46 +0200] rev 23721
added kind_of;
unparse: extra care for Malformed;
wenzelm [Tue, 10 Jul 2007 23:29:44 +0200] rev 23720
Markup.enclose;
wenzelm [Tue, 10 Jul 2007 23:29:43 +0200] rev 23719
more markup for inner and outer syntax;
added enclose;
wenzelm [Tue, 10 Jul 2007 23:29:41 +0200] rev 23718
simplified funpow, untabify;
wenzelm [Tue, 10 Jul 2007 23:29:38 +0200] rev 23717
added Thy/thy_edit.ML;
wenzelm [Tue, 10 Jul 2007 23:29:35 +0200] rev 23716
added some markup for outer syntax;
haftmann [Tue, 10 Jul 2007 17:30:57 +0200] rev 23715
clarified merge of module names
haftmann [Tue, 10 Jul 2007 17:30:56 +0200] rev 23714
now a monolithic module
haftmann [Tue, 10 Jul 2007 17:30:54 +0200] rev 23713
now works with SML/NJ
haftmann [Tue, 10 Jul 2007 17:30:53 +0200] rev 23712
tuned
haftmann [Tue, 10 Jul 2007 17:30:52 +0200] rev 23711
improvement for code names
haftmann [Tue, 10 Jul 2007 17:30:51 +0200] rev 23710
removed proof dependency on transitivity theorems
haftmann [Tue, 10 Jul 2007 17:30:50 +0200] rev 23709
moved lfp_induct2 here
haftmann [Tue, 10 Jul 2007 17:30:49 +0200] rev 23708
clarified import
haftmann [Tue, 10 Jul 2007 17:30:47 +0200] rev 23707
moved lfp_induct2 to Relation.thy
haftmann [Tue, 10 Jul 2007 17:30:45 +0200] rev 23706
moved some finite lemmas here
haftmann [Tue, 10 Jul 2007 17:30:43 +0200] rev 23705
moved finite lemmas to Finite_Set.thy
wenzelm [Tue, 10 Jul 2007 16:46:37 +0200] rev 23704
added print_mode setup (from pretty.ML);
removed no_state;
wenzelm [Tue, 10 Jul 2007 16:45:06 +0200] rev 23703
Markup.add_mode;
wenzelm [Tue, 10 Jul 2007 16:45:05 +0200] rev 23702
removed no_state markup -- produce empty state;
Markup.add_mode;
wenzelm [Tue, 10 Jul 2007 16:45:04 +0200] rev 23701
Markup.output;
removed no_state markup -- produce empty state;
wenzelm [Tue, 10 Jul 2007 16:45:03 +0200] rev 23700
moved source cascading from scan.ML to source.ML;
wenzelm [Tue, 10 Jul 2007 16:45:01 +0200] rev 23699
infixr || (more efficient);
tuned signature;
removed unused trace';
moved source cascading from scan.ML to source.ML;
tuned;
wenzelm [Tue, 10 Jul 2007 16:45:00 +0200] rev 23698
moved print_mode setup for markup to markup.ML;
wenzelm [Tue, 10 Jul 2007 16:45:00 +0200] rev 23697
Markup.output;
wenzelm [Tue, 10 Jul 2007 16:44:58 +0200] rev 23696
use position.ML earlier;
aspinall [Tue, 10 Jul 2007 15:45:34 +0200] rev 23695
Add widthN to signature
wenzelm [Tue, 10 Jul 2007 13:12:53 +0200] rev 23694
cd ISABELLE_HOME/etc;
haftmann [Tue, 10 Jul 2007 09:24:43 +0200] rev 23693
adjusted
haftmann [Tue, 10 Jul 2007 09:24:14 +0200] rev 23692
updated keywords
haftmann [Tue, 10 Jul 2007 09:23:17 +0200] rev 23691
simplified, tuned
haftmann [Tue, 10 Jul 2007 09:23:16 +0200] rev 23690
re-expanded paths
haftmann [Tue, 10 Jul 2007 09:23:15 +0200] rev 23689
replaced code generator framework for reflected cooper
haftmann [Tue, 10 Jul 2007 09:23:14 +0200] rev 23688
expanded fragile proof
haftmann [Tue, 10 Jul 2007 09:23:13 +0200] rev 23687
extended - convers now basic lcm properties also
haftmann [Tue, 10 Jul 2007 09:23:12 +0200] rev 23686
constant dvd now in class target
haftmann [Tue, 10 Jul 2007 09:23:11 +0200] rev 23685
moved lemma zdvd_period here
haftmann [Tue, 10 Jul 2007 09:23:10 +0200] rev 23684
introduced (auxiliary) class dvd_mod for more convenient code generation
wenzelm [Tue, 10 Jul 2007 00:43:51 +0200] rev 23683
tuned;
wenzelm [Tue, 10 Jul 2007 00:17:52 +0200] rev 23682
nested source: explicit interactive flag for recover avoids duplicate errors;
wenzelm [Mon, 09 Jul 2007 23:12:51 +0200] rev 23681
tuned dead code;
wenzelm [Mon, 09 Jul 2007 23:12:49 +0200] rev 23680
use Position.file_of;
removed strange comments;
wenzelm [Mon, 09 Jul 2007 23:12:46 +0200] rev 23679
toplevel_source: interactive flag indicates intermittent error_msg;
nested source: error msg passed to recover;
tuned source positions;
wenzelm [Mon, 09 Jul 2007 23:12:45 +0200] rev 23678
Malformed token: error msg;
scan: explicit handling of malformed symbols from previous stage;
source: interactive flag indicates intermittent error_msg;
tuned;
wenzelm [Mon, 09 Jul 2007 23:12:44 +0200] rev 23677
adapted OuterLex/T.source;
wenzelm [Mon, 09 Jul 2007 23:12:42 +0200] rev 23676
scan: changed treatment of malformed symbols, passed to next stage;
tuned sym_explode;
wenzelm [Mon, 09 Jul 2007 23:12:40 +0200] rev 23675
nested source: error msg passed to recover;
wenzelm [Mon, 09 Jul 2007 23:12:38 +0200] rev 23674
tuned signature;
nested source: error msg passed to recover;
wenzelm [Mon, 09 Jul 2007 23:12:37 +0200] rev 23673
replaced name by file (unquoted);
str_of: markup;
misc cleanup;
wenzelm [Mon, 09 Jul 2007 23:12:36 +0200] rev 23672
moved Path.position to Position.path;
wenzelm [Mon, 09 Jul 2007 23:12:35 +0200] rev 23671
proper position markup;
added properties operation;
tuned;
wenzelm [Mon, 09 Jul 2007 23:12:31 +0200] rev 23670
use position.ML after pretty.ML;
wenzelm [Mon, 09 Jul 2007 23:12:29 +0200] rev 23669
removed target RAW-ProofGeneral (impractical to maintain);
wenzelm [Mon, 09 Jul 2007 22:40:57 +0200] rev 23668
declare: disallow quote (") in names;
wenzelm [Mon, 09 Jul 2007 22:37:48 +0200] rev 23667
removed legacy ML file;
fixed prems_conv;
wenzelm [Mon, 09 Jul 2007 22:06:49 +0200] rev 23666
HOL-Complex-Matrix: fixed deps -- sort of;
obua [Mon, 09 Jul 2007 17:39:55 +0200] rev 23665
adopted to new computing oracle and fixed bugs introduced by tuning
obua [Mon, 09 Jul 2007 17:38:40 +0200] rev 23664
added computing oracle support for HOL and numerals
obua [Mon, 09 Jul 2007 17:36:25 +0200] rev 23663
new version of computing oracle
wenzelm [Mon, 09 Jul 2007 11:44:23 +0200] rev 23662
simplified writeln_fn;
wenzelm [Mon, 09 Jul 2007 11:44:22 +0200] rev 23661
prompt: plain string, not output;
wenzelm [Mon, 09 Jul 2007 11:44:20 +0200] rev 23660
type output = string indicates raw system output;
wenzelm [Sun, 08 Jul 2007 19:52:10 +0200] rev 23659
symbolic output: avoid empty blocks, 1 space for fbreak;
wenzelm [Sun, 08 Jul 2007 19:52:08 +0200] rev 23658
tuned;
wenzelm [Sun, 08 Jul 2007 19:52:05 +0200] rev 23657
thm tag: Markup.property list;
wenzelm [Sun, 08 Jul 2007 19:52:04 +0200] rev 23656
gensym: slightly more obscure prefix descreases probability of name clash;
wenzelm [Sun, 08 Jul 2007 19:51:58 +0200] rev 23655
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
wenzelm [Sun, 08 Jul 2007 19:51:55 +0200] rev 23654
attribute tagged: single argument;
wenzelm [Sun, 08 Jul 2007 19:51:54 +0200] rev 23653
updated;
wenzelm [Sun, 08 Jul 2007 19:51:52 +0200] rev 23652
simplified Symtab;
wenzelm [Sun, 08 Jul 2007 19:51:51 +0200] rev 23651
renamed ML_exc to ML_exn;
chaieb [Sun, 08 Jul 2007 19:01:32 +0200] rev 23650
Show the use of reflection attribute; fixed comments about the order of absorbing equations : f (C x) = x ; now automaically tried as last;
chaieb [Sun, 08 Jul 2007 19:01:30 +0200] rev 23649
Changed syntax for the reflection method (reify unchanged). reflection takes an optional set of theorems for reification then several correctness theorems are specified by rules:'' then the optional term is specified by only:
chaieb [Sun, 08 Jul 2007 19:01:28 +0200] rev 23648
Try several correctness theorems for reflection; rearrange cong rules to avoid the absoption cases;
chaieb [Sun, 08 Jul 2007 19:01:26 +0200] rev 23647
Context data now consist of eqations for reification and equations for correctness theorems for reflection; Added attribute reflection to store correctness theorems to be trued by default
wenzelm [Sun, 08 Jul 2007 13:10:57 +0200] rev 23646
simplified/more robust print_state;
more robust prompt markup;
wenzelm [Sun, 08 Jul 2007 13:10:54 +0200] rev 23645
export mode_markup;
added symbolic output (via print_mode);
misc cleanup;
wenzelm [Sun, 08 Jul 2007 13:10:51 +0200] rev 23644
added markup for pretty printing;
chaieb [Sun, 08 Jul 2007 12:20:56 +0200] rev 23643
Corrected erronus use of compiletime context to the runtime context
wenzelm [Sat, 07 Jul 2007 18:47:47 +0200] rev 23642
make smlnj happy;
wenzelm [Sat, 07 Jul 2007 18:39:21 +0200] rev 23641
toplevel prompt/print_state: proper markup, removed hooks;
wenzelm [Sat, 07 Jul 2007 18:39:20 +0200] rev 23640
toplevel prompt/print_state: proper markup, removed hooks;
tuned;
wenzelm [Sat, 07 Jul 2007 18:39:19 +0200] rev 23639
pretty_state: subgoal markup;
tuned;
wenzelm [Sat, 07 Jul 2007 18:39:18 +0200] rev 23638
added markup_chunks;
wenzelm [Sat, 07 Jul 2007 18:39:17 +0200] rev 23637
added toplevel markup;
misc cleanup;
wenzelm [Sat, 07 Jul 2007 18:39:16 +0200] rev 23636
use markup.ML earlier;
wenzelm [Sat, 07 Jul 2007 18:39:15 +0200] rev 23635
removed obsolete disable_pr/enable_pr;
added old print_goals from display.ML;
wenzelm [Sat, 07 Jul 2007 18:39:14 +0200] rev 23634
pretty_goals_aux: subgoal markup;
print_goals etc.: moved old version to old_goals.ML, removed hooks;
tuned;
wenzelm [Sat, 07 Jul 2007 18:39:12 +0200] rev 23633
pr_goals: adapted Display.pretty_goals_aux;
pr_goals/prterm: proper context;
tuned;
wenzelm [Sat, 07 Jul 2007 12:16:20 +0200] rev 23632
export attribute;
wenzelm [Sat, 07 Jul 2007 12:16:19 +0200] rev 23631
pretty_sort/typ/term: markup;
wenzelm [Sat, 07 Jul 2007 12:16:18 +0200] rev 23630
pretty: markup for syntax/name of authentic consts;
datatype symb: String (potential markup) vs. Space (no markup);
wenzelm [Sat, 07 Jul 2007 12:16:17 +0200] rev 23629
depend on alist.ML, markup.ML;
wenzelm [Sat, 07 Jul 2007 12:16:16 +0200] rev 23628
markup: emit as control information -- no indent text;
wenzelm [Sat, 07 Jul 2007 12:16:15 +0200] rev 23627
added property conversions;
tuned;
wenzelm [Sat, 07 Jul 2007 12:16:14 +0200] rev 23626
position: line and name;
tuned operations;
wenzelm [Sat, 07 Jul 2007 12:16:13 +0200] rev 23625
moved markup.ML before position.ML;
chaieb [Sat, 07 Jul 2007 11:09:40 +0200] rev 23624
The order for parameter for interpretation is now inversted:
f t env0 env1 ... envn = ...
where t is the type to be reified;
wenzelm [Sat, 07 Jul 2007 00:17:10 +0200] rev 23623
Common markup elements.
wenzelm [Sat, 07 Jul 2007 00:15:03 +0200] rev 23622
simplified pretty token metric: type int;
added command markup;
token translations: proper treatment of skolems;
separate print_mode setup for Output/Pretty;
wenzelm [Sat, 07 Jul 2007 00:15:02 +0200] rev 23621
simplified pretty token metric: type int;
separate print_mode setup for Output/Pretty;
wenzelm [Sat, 07 Jul 2007 00:15:02 +0200] rev 23620
moved General/xml.ML to Tools/xml.ML;
actually use pgml.ML;
wenzelm [Sat, 07 Jul 2007 00:15:00 +0200] rev 23619
tuned;
wenzelm [Sat, 07 Jul 2007 00:14:59 +0200] rev 23618
simplified output mode setup;
removed unused symbol_output;
tuned;
wenzelm [Sat, 07 Jul 2007 00:14:58 +0200] rev 23617
added print_mode setup: indent and markup;
simplified pretty token metric: type int;
added general markup for blocks;
removed unused writelns;
wenzelm [Sat, 07 Jul 2007 00:14:57 +0200] rev 23616
renamed raw to escape;
simplified pretty token metric: type int;
simplified print_mode setup: output_width and escape;
moved pretty setup to pretty.ML;
wenzelm [Sat, 07 Jul 2007 00:14:56 +0200] rev 23615
simplified pretty token metric: type int;
wenzelm [Sat, 07 Jul 2007 00:14:54 +0200] rev 23614
moved General/xml.ML to Tools/xml.ML;
wenzelm [Sat, 07 Jul 2007 00:14:52 +0200] rev 23613
added General/markup.ML;
moved General/xml.ML to Tools/xml.ML;
wenzelm [Sat, 07 Jul 2007 00:14:49 +0200] rev 23612
added class skolem, command;
nipkow [Fri, 06 Jul 2007 23:26:13 +0200] rev 23611
more interpretations
aspinall [Fri, 06 Jul 2007 17:52:52 +0200] rev 23610
Produce good PGML 2.0
webertj [Fri, 06 Jul 2007 17:21:18 +0200] rev 23609
cosmetic (line length fixed)
chaieb [Fri, 06 Jul 2007 16:09:28 +0200] rev 23608
Some examples for reifying type variables
chaieb [Fri, 06 Jul 2007 16:09:27 +0200] rev 23607
Tuned document
chaieb [Fri, 06 Jul 2007 16:09:26 +0200] rev 23606
Cleaned add and del attributes
chaieb [Fri, 06 Jul 2007 16:09:25 +0200] rev 23605
Reification now deals with type variables
wenzelm [Fri, 06 Jul 2007 11:55:05 +0200] rev 23604
Cumulative reports for Poly/ML profiling output.
aspinall [Thu, 05 Jul 2007 20:36:48 +0200] rev 23603
Update PGML version, add system name
wenzelm [Thu, 05 Jul 2007 20:01:39 +0200] rev 23602
tuned interfaces: atomize, atomize_prems, atomize_prems_tac;
removed atomize_cterm/goal;
wenzelm [Thu, 05 Jul 2007 20:01:38 +0200] rev 23601
added type conv;
merge_thys: removed dead exception handlers;
tuned;
wenzelm [Thu, 05 Jul 2007 20:01:37 +0200] rev 23600
removed comments -- no exception TERM;
merge_list: exception THEORY;
wenzelm [Thu, 05 Jul 2007 20:01:36 +0200] rev 23599
added is_reflexive;
wenzelm [Thu, 05 Jul 2007 20:01:35 +0200] rev 23598
tuned;
wenzelm [Thu, 05 Jul 2007 20:01:34 +0200] rev 23597
simplified has_meta_prems;
wenzelm [Thu, 05 Jul 2007 20:01:33 +0200] rev 23596
moved type conv to thm.ML;
renamed Conv.is_refl to Thm.is_reflexive;
misc tuning of basic conversions;
wenzelm [Thu, 05 Jul 2007 20:01:32 +0200] rev 23595
the_theory/proof: error instead of exception Fail;
wenzelm [Thu, 05 Jul 2007 20:01:31 +0200] rev 23594
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
added flat_rule filter for addXXs etc.;
wenzelm [Thu, 05 Jul 2007 20:01:30 +0200] rev 23593
renamed Conv.is_refl to Thm.is_reflexive;
wenzelm [Thu, 05 Jul 2007 20:01:29 +0200] rev 23592
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
simplified ObjectLogic.atomize;
wenzelm [Thu, 05 Jul 2007 20:01:28 +0200] rev 23591
simplified ObjectLogic.atomize;
wenzelm [Thu, 05 Jul 2007 20:01:26 +0200] rev 23590
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
aspinall [Thu, 05 Jul 2007 19:59:01 +0200] rev 23589
Revert body of pgml to match schema for now [change bad for Broker]
aspinall [Thu, 05 Jul 2007 19:57:19 +0200] rev 23588
Classify -- comments as ordinary comments (no undo)
wenzelm [Thu, 05 Jul 2007 00:15:44 +0200] rev 23587
tuned;
wenzelm [Thu, 05 Jul 2007 00:06:25 +0200] rev 23586
avoid polymorphic equality;
added dest_judgment;
wenzelm [Thu, 05 Jul 2007 00:06:24 +0200] rev 23585
sort_le: tuned eq case;
wenzelm [Thu, 05 Jul 2007 00:06:23 +0200] rev 23584
tuned goal conversion interfaces;
wenzelm [Thu, 05 Jul 2007 00:06:22 +0200] rev 23583
else_conv: only handle THM | CTERM | TERM | TYPE;
prems_conv: no index;
renamed goal_conv_rule to gconv_rule;
wenzelm [Thu, 05 Jul 2007 00:06:20 +0200] rev 23582
avoid polymorphic equality;
Numeral.mk_cnumber;
wenzelm [Thu, 05 Jul 2007 00:06:19 +0200] rev 23581
tuned;
wenzelm [Thu, 05 Jul 2007 00:06:18 +0200] rev 23580
moved mk_cnumeral/mk_cnumber to Tools/numeral.ML;
tuned;
wenzelm [Thu, 05 Jul 2007 00:06:17 +0200] rev 23579
avoid polymorphic equality;
do not export ring_conv (which is not a conversion anyway);
renamed algebra_tac to ring_tac;
ring_tac: simplified tactic wrapper, no longer handles ERROR;
wenzelm [Thu, 05 Jul 2007 00:06:16 +0200] rev 23578
avoid polymorphic equality;
removed dead code;
wenzelm [Thu, 05 Jul 2007 00:06:14 +0200] rev 23577
avoid polymorphic equality;
wenzelm [Thu, 05 Jul 2007 00:06:13 +0200] rev 23576
removed dest_cTrueprop (cf. ObjectLogic.dest_judgment);
wenzelm [Thu, 05 Jul 2007 00:06:12 +0200] rev 23575
Logical operations on numerals (see also HOL/hologic.ML).
wenzelm [Thu, 05 Jul 2007 00:06:11 +0200] rev 23574
added Tools/numeral.ML;
wenzelm [Thu, 05 Jul 2007 00:06:10 +0200] rev 23573
common normalizer_funs, avoid cterm_of;
wenzelm [Thu, 05 Jul 2007 00:06:09 +0200] rev 23572
Numeral.mk_cnumber;
aspinall [Wed, 04 Jul 2007 21:20:23 +0200] rev 23571
PGML abstraction, draft version
aspinall [Wed, 04 Jul 2007 21:19:34 +0200] rev 23570
Use pgml
obua [Wed, 04 Jul 2007 17:21:02 +0200] rev 23569
fixed argument order in calls to Integer.pow
wenzelm [Wed, 04 Jul 2007 16:49:36 +0200] rev 23568
added binop_cong_rule;
wenzelm [Wed, 04 Jul 2007 16:49:35 +0200] rev 23567
export dlo_conv;
removed redundant auxiliary operations;
tuned exceptions -- avoid error here;
simplified tactic wrapper (CSUBGOAL, CONVERSION);
merge_ss: recover simpset context;
tuned;
wenzelm [Wed, 04 Jul 2007 16:49:34 +0200] rev 23566
replaced HOLogic.Trueprop_conv by ObjectLogic.judgment_conv;
nipkow [Wed, 04 Jul 2007 14:21:00 +0200] rev 23565
*** empty log message ***
nipkow [Wed, 04 Jul 2007 14:10:01 +0200] rev 23564
*** empty log message ***
paulson [Wed, 04 Jul 2007 13:56:26 +0200] rev 23563
simplified a proof
wenzelm [Tue, 03 Jul 2007 23:00:42 +0200] rev 23562
tuned;
wenzelm [Tue, 03 Jul 2007 22:27:30 +0200] rev 23561
CONVERSION: handle TYPE | TERM | CTERM | THM;
wenzelm [Tue, 03 Jul 2007 22:27:27 +0200] rev 23560
proper use of ioa_package.ML;
wenzelm [Tue, 03 Jul 2007 22:27:25 +0200] rev 23559
tuned;
wenzelm [Tue, 03 Jul 2007 22:27:19 +0200] rev 23558
tuned is_comb/is_binop -- avoid construction of cterms;
removed conjunction rules (cf. HOLogic.conj_XXX);
wenzelm [Tue, 03 Jul 2007 22:27:16 +0200] rev 23557
HOLogic.conj_intr/elims;
removed obsolete assocd/assoc;
removed dead string_of_pol;
tuned;
wenzelm [Tue, 03 Jul 2007 22:27:13 +0200] rev 23556
use mucke_oracle.ML only once;
wenzelm [Tue, 03 Jul 2007 22:27:11 +0200] rev 23555
assume basic HOL context for compilation (antiquotations);
added dest_cTrueprop;
tuned Trueprop_conv;
added low-level conj_intr/elim/elis (dire need for @{rule} antiquotation!);
wenzelm [Tue, 03 Jul 2007 22:27:08 +0200] rev 23554
proper use of function_package ML files;
wenzelm [Tue, 03 Jul 2007 22:27:05 +0200] rev 23553
use hologic.ML in basic HOL context;
tuned proofs;
paulson [Tue, 03 Jul 2007 21:56:25 +0200] rev 23552
to handle non-atomic assumptions
wenzelm [Tue, 03 Jul 2007 20:26:08 +0200] rev 23551
rename class dom to ring_1_no_zero_divisors (cf. HOL/Ring_and_Field.thy 1.84 by huffman);
huffman [Tue, 03 Jul 2007 18:42:09 +0200] rev 23550
convert instance proofs to Isar style
chaieb [Tue, 03 Jul 2007 18:00:57 +0200] rev 23549
Dependency on reflection_data.ML to build HOL-ex
chaieb [Tue, 03 Jul 2007 17:50:00 +0200] rev 23548
Generalized case for atoms. Selection of environment lists is allowed more than once.
chaieb [Tue, 03 Jul 2007 17:49:58 +0200] rev 23547
More examples
chaieb [Tue, 03 Jul 2007 17:49:55 +0200] rev 23546
reflection and reification methods now manage Context data
chaieb [Tue, 03 Jul 2007 17:49:53 +0200] rev 23545
Context Data for the reflection and reification methods
huffman [Tue, 03 Jul 2007 17:28:36 +0200] rev 23544
rename class dom to ring_1_no_zero_divisors
wenzelm [Tue, 03 Jul 2007 17:17:17 +0200] rev 23543
rewrite_goal_tac;
wenzelm [Tue, 03 Jul 2007 17:17:16 +0200] rev 23542
replaced Conv.goals_conv by Conv.prems_conv;
wenzelm [Tue, 03 Jul 2007 17:17:15 +0200] rev 23541
exported meta_rewrite_conv;
CONVERSION tactical;