src/HOL/ex/Locales.thy
changeset 13419 902ec83c1ca9
parent 13383 041d78bf9403
child 13457 7ddcf40a80b3
equal deleted inserted replaced
13418:7c0ba9dba978 13419:902ec83c1ca9
   231   contexts is rather light-weight and convenient to use for abstract
   231   contexts is rather light-weight and convenient to use for abstract
   232   reasoning.  Here the ``components'' (the group operations) have been
   232   reasoning.  Here the ``components'' (the group operations) have been
   233   exhibited directly as context parameters; logically this corresponds
   233   exhibited directly as context parameters; logically this corresponds
   234   to a curried predicate definition:
   234   to a curried predicate definition:
   235 
   235 
   236   @{thm [display] group_context_axioms_def [no_vars]}
   236   @{thm [display] group_context_def [no_vars]}
       
   237 
       
   238   The corresponding introduction rule is as follows:
       
   239 
       
   240   @{thm [display] group_context.intro [no_vars]}
   237 
   241 
   238   Occasionally, this ``externalized'' version of the informal idea of
   242   Occasionally, this ``externalized'' version of the informal idea of
   239   classes of tuple structures may cause some inconveniences,
   243   classes of tuple structures may cause some inconveniences,
   240   especially in meta-theoretical studies (involving functors from
   244   especially in meta-theoretical studies (involving functors from
   241   groups to groups, for example).
   245   groups to groups, for example).